Skip to content

Commit

Permalink
Remove fterm internals from the CClosure API.
Browse files Browse the repository at this point in the history
  • Loading branch information
ppedrot committed Dec 19, 2024
1 parent a158888 commit 9d01c8e
Show file tree
Hide file tree
Showing 2 changed files with 0 additions and 9 deletions.
3 changes: 0 additions & 3 deletions kernel/cClosure.ml
Original file line number Diff line number Diff line change
Expand Up @@ -114,9 +114,6 @@ let get_invert fiv = fiv
let fterm_of v = v.term
let set_ntrl v = v.mark <- Ntrl

let mk_atom c = {mark=Ntrl;term=FAtom c}
let mk_red f = {mark=Red;term=f}

(* Could issue a warning if no is still Red, pointing out that we loose
sharing. *)
let update v1 mark t =
Expand Down
6 changes: 0 additions & 6 deletions kernel/cClosure.mli
Original file line number Diff line number Diff line change
Expand Up @@ -108,12 +108,6 @@ val inject : constr -> fconstr
val mk_clos : usubs -> constr -> fconstr
val mk_clos_vect : usubs -> constr array -> fconstr array

(** mk_atom: prevents a term from being evaluated *)
val mk_atom : constr -> fconstr

(** mk_red: makes a reducible term (used in ring) *)
val mk_red : fterm -> fconstr

val zip : fconstr -> stack -> fconstr

val fterm_of : fconstr -> fterm
Expand Down

0 comments on commit 9d01c8e

Please sign in to comment.