Skip to content

Commit

Permalink
Split Logic into subdirectories
Browse files Browse the repository at this point in the history
  • Loading branch information
proux01 committed Sep 21, 2024
1 parent 0ff3c4e commit 0d98057
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion library/coqlib.ml
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,7 @@ let coq = Libnames.coq_string (* "Stdlib" *)

let init_dir = [ coq; "Init"]

let jmeq_module_name = [coq;"Logic";"JMeq"]
let jmeq_module_name = [coq;"Logic";"Base"; "Stdlib"; "Logic"; "JMeq"]

let find_reference locstr dir s =
let dp = make_dir dir in
Expand Down
2 changes: 1 addition & 1 deletion pretyping/program.ml
Original file line number Diff line number Diff line change
Expand Up @@ -44,7 +44,7 @@ let mk_coq_not env sigma x =
let coq_JMeq_ind () =
try Coqlib.lib_ref "core.JMeq.type"
with Not_found ->
user_err (Pp.str "cannot find Stdlib.Logic.JMeq.JMeq; maybe library Stdlib.Logic.JMeq has to be required first.")
user_err (Pp.str "cannot find Stdlib.Logic.Base.Stdlib.Logic.JMeq.JMeq; maybe library JMeq from Stdlib has to be required first.")
let coq_JMeq_refl () = Coqlib.lib_ref "core.JMeq.refl"

(* let coq_not () = Universes.constr_of_global @@ Coqlib.lib_ref "core.not.type" *)
Expand Down

0 comments on commit 0d98057

Please sign in to comment.