diff options
| author | Arnaud Spiwack | 2015-03-12 17:32:50 +0100 |
|---|---|---|
| committer | Arnaud Spiwack | 2015-03-13 16:41:03 +0100 |
| commit | 71fcb53fd93edcac1925f97d619871e8597e24e2 (patch) | |
| tree | 5d4a197262c3ba8d86f6127ed2cd98a896d45130 /plugins | |
| parent | caa1e9278136bbf2c9353eeb415d331eee99c172 (diff) | |
Declarative mode: remove dead code.
Diffstat (limited to 'plugins')
| -rw-r--r-- | plugins/decl_mode/decl_mode.ml | 3 | ||||
| -rw-r--r-- | plugins/decl_mode/decl_mode.mli | 2 |
2 files changed, 0 insertions, 5 deletions
diff --git a/plugins/decl_mode/decl_mode.ml b/plugins/decl_mode/decl_mode.ml index 07bf6d3268..da41cd86db 100644 --- a/plugins/decl_mode/decl_mode.ml +++ b/plugins/decl_mode/decl_mode.ml @@ -105,9 +105,6 @@ let focus p = let unfocus () = Proof_global.simple_with_current_proof (fun _ p -> Proof.unfocus proof_focus p ()) -let maximal_unfocus () = - Proof_global.simple_with_current_proof (fun _ -> Proof.maximal_unfocus proof_focus) - let get_top_stack pts = try Proof.get_at_focus proof_focus pts diff --git a/plugins/decl_mode/decl_mode.mli b/plugins/decl_mode/decl_mode.mli index 2864ba18ee..e12c4c9237 100644 --- a/plugins/decl_mode/decl_mode.mli +++ b/plugins/decl_mode/decl_mode.mli @@ -75,5 +75,3 @@ val get_last: Environ.env -> Id.t val focus : Proof.proof -> unit val unfocus : unit -> unit - -val maximal_unfocus : unit -> unit |
