diff options
| author | letouzey | 2012-10-02 15:58:00 +0000 |
|---|---|---|
| committer | letouzey | 2012-10-02 15:58:00 +0000 |
| commit | 85c509a0fada387d3af96add3dac6a7c702b5d01 (patch) | |
| tree | 4d262455aed52c20af0a9627d47d29b03ca6523d /plugins/decl_mode | |
| parent | 3415801b2c368ce03f6e8d33a930b9ab9e0b9fd1 (diff) | |
Remove some more "open" and dead code thanks to OCaml4 warnings
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15844 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/decl_mode')
| -rw-r--r-- | plugins/decl_mode/decl_mode.ml | 1 | ||||
| -rw-r--r-- | plugins/decl_mode/decl_proof_instr.ml | 17 | ||||
| -rw-r--r-- | plugins/decl_mode/g_decl_mode.ml4 | 3 | ||||
| -rw-r--r-- | plugins/decl_mode/ppdecl_proof.ml | 1 |
4 files changed, 0 insertions, 22 deletions
diff --git a/plugins/decl_mode/decl_mode.ml b/plugins/decl_mode/decl_mode.ml index f29964c69e..1f55257e5e 100644 --- a/plugins/decl_mode/decl_mode.ml +++ b/plugins/decl_mode/decl_mode.ml @@ -12,7 +12,6 @@ open Evd open Errors open Util - let daimon_flag = ref false let set_daimon_flag () = daimon_flag:=true diff --git a/plugins/decl_mode/decl_proof_instr.ml b/plugins/decl_mode/decl_proof_instr.ml index 1a0d05047e..367e02bf8e 100644 --- a/plugins/decl_mode/decl_proof_instr.ml +++ b/plugins/decl_mode/decl_proof_instr.ml @@ -11,7 +11,6 @@ open Util open Pp open Evd -open Proof_type open Tacmach open Tacinterp open Decl_expr @@ -129,22 +128,6 @@ let daimon_tac gls = set_daimon_flag (); {it=[];sigma=sig_sig gls} - -(* marking closed blocks *) - -let rec is_focussing_instr = function - Pthus i | Pthen i | Phence i -> is_focussing_instr i - | Pescape | Pper _ | Pclaim _ | Pfocus _ - | Psuppose _ | Pcase (_,_,_) -> true - | _ -> false - -let mark_rule_as_done = function - Decl_proof true -> Decl_proof false - | Decl_proof false -> - anomaly "already marked as done" - | _ -> anomaly "mark_rule_as_done" - - (* post-instruction focus management *) (* spiwack: This used to fail if there was no focusing command diff --git a/plugins/decl_mode/g_decl_mode.ml4 b/plugins/decl_mode/g_decl_mode.ml4 index 3eaf81d2bc..e8e81c472c 100644 --- a/plugins/decl_mode/g_decl_mode.ml4 +++ b/plugins/decl_mode/g_decl_mode.ml4 @@ -14,13 +14,10 @@ open Pp open Tok open Decl_expr open Names -open Term -open Genarg open Pcoq open Pcoq.Constr open Pcoq.Tactic -open Pcoq.Vernac_ let pr_goal gs = let (g,sigma) = Goal.V82.nf_evar (Tacmach.project gs) (Evd.sig_it gs) in diff --git a/plugins/decl_mode/ppdecl_proof.ml b/plugins/decl_mode/ppdecl_proof.ml index b72476a756..01f32e4a32 100644 --- a/plugins/decl_mode/ppdecl_proof.ml +++ b/plugins/decl_mode/ppdecl_proof.ml @@ -7,7 +7,6 @@ (************************************************************************) open Errors -open Util open Pp open Decl_expr open Names |
