HOL icon indicating copy to clipboard operation
HOL copied to clipboard

Canonical sources for HOL4 theorem-proving system. Branch develop is where “mainline development” occurs; when develop passes our regression tests, master is merged forward to catch up.

Results 138 HOL issues
Sort by recently updated
recently updated
newest added

Following commit f6c3ef2, loading intLib produces a lot of output that should be suppressed and/or avoided (see below). Ideally there should not be calls to Meson when loading the library....

Tactics/DPs

Hi, This PR ports the ring decision procedure (`RING_TAC` and `RING_RULE`) from HOL-Light ([`ringtheory.ml`](https://github.com/jrh13/hol-light/blob/master/Library/ringtheory.ml)). The ring decision procedure, currently located at `examples/algebra/ring/ringLib.sml`, can be used to decide equations about ring...

I think this issue is new on macOS 14 (Sonoma) with latest Xcode (I'm using version 15.3). Apple's `c++` (`clang++`) cannot compile `src/HolSat/sat_solvers/zc2hs/zc2hs.cpp`: ``` src/HolSat/sat_solvers/zc2hs$ make ln -fs ../minisat/Proof.o ln...

Hi, It seems that for each core theory there are two HTML pages generated in the help page. One is that you directly click the theory names from the HOL...

`Q.PAT_X_ASSUM` (_aka_ `qpat_x_assum`) returns bad error messages because its implementation can't distinguish between an expected failure (the pattern not matching an unrelated assumption) and an unexpected failure (the continuation failing)....

Feature Request
Tactics/DPs

Suggestion from @myreen on Discord: > Could there be general-purpose quote filter support for making this nicer? Specifics can be discussed, but something along these lines: ``` val cakeml_code =...

Printing-Parsing
Feature Request

Can be useful to match on a sub-term of an assumption.

Feature Request
Tactics/DPs

It should be possible to specialise variables without knowing where in a quantification block they are, and if free, the effect can be as of `INST`.

Feature Request

Something like ``` simp[IgnAsm ‘pat’, th1] ``` should apply the simplifier, while ignoring the assumption(s) matching `pat`. Also ``` simp[NoAsms,...] ``` should ignore all assumptions.

Simplifier
Feature Request

I'm running into an issue where both `intLib.ARITH_PROVE` and `intLib.COOPER_PROVE` are failing to prove certain goals, even though it seems like they should be able to handle them. Here are...