diff options
author | Enrico Tassi <enrico.tassi@inria.fr> | 2015-03-09 18:44:33 +0100 |
---|---|---|
committer | Enrico Tassi <enrico.tassi@inria.fr> | 2015-03-11 11:42:10 +0100 |
commit | f36f1d07ee0b9b40d54b9fece942b00e8e5e5d50 (patch) | |
tree | 4b3d9cf2a0ed1ef4faa1d6bfccaaf0ca878a942d /plugins/derive | |
parent | e4ad47fed594d6865f5bd29a159976cb072f0fae (diff) |
admit: replaced by give_up + Admitted (no proof_admitted : False, close #4032)
- no more inconsistent Axiom in the Prelude
- STM can now process Admitted proofs asynchronously
- the quick chain can stock "Admitted" jobs in .vio files
- the vio2vo step checks the jobs but does not stock the result
in the opaque tables (they have no slot)
- Admitted emits a warning if the proof is complete
- Admitted uses the (partial) proof term to infer section variables
used (if not given with Proof using), like for Qed
- test-suite: extra line Require TestSuite.admit to each file making
use of admit
- test-suite/_CoqProject: to pass to CoqIDE and PG the right -Q flag to
find TestSuite.admit
Diffstat (limited to 'plugins/derive')
-rw-r--r-- | plugins/derive/derive.ml | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/derive/derive.ml b/plugins/derive/derive.ml index a77b552e0..c232ae31a 100644 --- a/plugins/derive/derive.ml +++ b/plugins/derive/derive.ml @@ -49,7 +49,7 @@ let start_deriving f suchthat lemma = [suchthat], respectively. *) let (opaque,f_def,lemma_def) = match com with - | Admitted -> Errors.error"Admitted isn't supported in Derive." + | Admitted _ -> Errors.error"Admitted isn't supported in Derive." | Proved (_,Some _,_) -> Errors.error"Cannot save a proof of Derive with an explicit name." | Proved (opaque, None, obj) -> |