aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2020-06-26 12:56:26 +0200
committerPierre-Marie Pédrot2020-06-29 15:20:37 +0200
commita33f772631696c694f0d9a7fad3a914037c464b2 (patch)
tree0f7c0f9c3d363f13d0d5d28a67281e7547f7a3db
parentd28af587b9848c6155c7eae482591836f0fbc68f (diff)
Refining out the Refiner.
-rw-r--r--dev/base_include1
-rw-r--r--proofs/proofs.mllib1
-rw-r--r--proofs/refiner.ml9
-rw-r--r--proofs/refiner.mli11
4 files changed, 0 insertions, 22 deletions
diff --git a/dev/base_include b/dev/base_include
index 67ea3a1fa1..1f14fc2941 100644
--- a/dev/base_include
+++ b/dev/base_include
@@ -114,7 +114,6 @@ open Logic
open Proof
open Proof_using
open Redexpr
-open Refiner
open Tacmach
open Hints
diff --git a/proofs/proofs.mllib b/proofs/proofs.mllib
index 790a9dd2cc..5f19c1bb09 100644
--- a/proofs/proofs.mllib
+++ b/proofs/proofs.mllib
@@ -6,6 +6,5 @@ Proof
Logic
Goal_select
Proof_bullet
-Refiner
Tacmach
Clenv
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
deleted file mode 100644
index b72d544151..0000000000
--- a/proofs/refiner.ml
+++ /dev/null
@@ -1,9 +0,0 @@
-(************************************************************************)
-(* * The Coq Proof Assistant / The Coq Development Team *)
-(* v * Copyright INRIA, CNRS and contributors *)
-(* <O___,, * (see version control and CREDITS file for authors & dates) *)
-(* \VV/ **************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(* * (see LICENSE file for the text of the license) *)
-(************************************************************************)
diff --git a/proofs/refiner.mli b/proofs/refiner.mli
deleted file mode 100644
index c38cb23cb0..0000000000
--- a/proofs/refiner.mli
+++ /dev/null
@@ -1,11 +0,0 @@
-(************************************************************************)
-(* * The Coq Proof Assistant / The Coq Development Team *)
-(* v * Copyright INRIA, CNRS and contributors *)
-(* <O___,, * (see version control and CREDITS file for authors & dates) *)
-(* \VV/ **************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(* * (see LICENSE file for the text of the license) *)
-(************************************************************************)
-
-(** Legacy proof engine. Do not use in newly written code. *)