Skip to content

Commit

Permalink
Remove Summary.Local (deprecated in 8.18)
Browse files Browse the repository at this point in the history
  • Loading branch information
SkySkimmer committed Oct 26, 2023
1 parent 1cbd585 commit 0c15794
Show file tree
Hide file tree
Showing 3 changed files with 1 addition and 21 deletions.
10 changes: 0 additions & 10 deletions library/summary.ml
Original file line number Diff line number Diff line change
Expand Up @@ -216,14 +216,4 @@ let ref ?(stage=Stage.Interp) ?(local=false) ~name x =
in
r

module Local = struct

type 'a local_ref = 'a ref

let ref ?stage ~name x = ref ?stage ~name ~local:true x
let (!) = (!)
let (:=) = (:=)

end

let dump = Dyn.dump
9 changes: 0 additions & 9 deletions library/summary.mli
Original file line number Diff line number Diff line change
Expand Up @@ -67,15 +67,6 @@ val declare_summary_tag : string -> ?make_marshallable:('a -> 'a) -> 'a summary_
val ref : ?stage:Stage.t -> ?local:bool -> name:string -> 'a -> 'a ref
val ref_tag : ?stage:Stage.t -> name:string -> 'a -> 'a ref * 'a Dyn.tag

module Local : sig

type 'a local_ref = 'a ref
val ref : ?stage:Stage.t -> name:string -> 'a -> 'a local_ref
val (:=) : 'a local_ref -> 'a -> unit
val (!) : 'a local_ref -> 'a

end [@@ocaml.deprecated "Use [Summary.ref ~local:true]"]

(** Special summary for ML modules. This summary entry is special
because its unfreeze may load ML code and hence add summary
entries. Thus is has to be recognizable, and handled properly.
Expand Down
3 changes: 1 addition & 2 deletions test-suite/misc/non-marshalable-state/src/good.mlg
Original file line number Diff line number Diff line change
Expand Up @@ -2,15 +2,14 @@ DECLARE PLUGIN "coq-test-suite.good"

{

let state = Summary.Local.ref
let state = Summary.ref ~local:true
~name:"elpi-compiler-cache"
None

}

VERNAC COMMAND EXTEND magic CLASSIFIED AS SIDEFF
| [ "magic" ] -> {
let open Summary.Local in
state := Some (fun () -> ())
}
END

0 comments on commit 0c15794

Please sign in to comment.