diff options
author | Pierre Letouzey <pierre.letouzey@inria.fr> | 2016-06-23 15:07:02 +0200 |
---|---|---|
committer | Pierre Letouzey <pierre.letouzey@inria.fr> | 2017-06-14 12:02:35 +0200 |
commit | 27c8e30fad95d887b698b0e3fa563644c293b033 (patch) | |
tree | 021febbccb12aff7873cf18aebaf4e9e2a6e4d47 /test-suite/ide | |
parent | b240771a3661883ca0cc0497efee5b48519bddea (diff) |
Prelude : no more autoload of plugins extraction and recdef
The user now has to manually load them, respectively via:
Require Extraction
Require Import FunInd
The "Import" in the case of FunInd is to ensure that the
tactics functional induction and functional inversion are indeed
in scope.
Note that the Recdef.v file is still there as well (it contains
complements used when doing Function with measures), and it also
triggers a load of FunInd.v.
This change is correctly documented in the refman, and the test-suite
has been adapted.
Diffstat (limited to 'test-suite/ide')
-rw-r--r-- | test-suite/ide/blocking-futures.fake | 1 |
1 files changed, 1 insertions, 0 deletions
diff --git a/test-suite/ide/blocking-futures.fake b/test-suite/ide/blocking-futures.fake index b63f09bcf..541fb798c 100644 --- a/test-suite/ide/blocking-futures.fake +++ b/test-suite/ide/blocking-futures.fake @@ -4,6 +4,7 @@ # Extraction will force the future computation, assert it is blocking # Example courtesy of Jonathan (jonikelee) # +ADD { Require Coq.extraction.Extraction. } ADD { Require Import List. } ADD { Import ListNotations. } ADD { Definition myrev{A}(l : list A) : {rl : list A | rl = rev l}. } |