Skip to content

Commit

Permalink
[ringLib] RING_TAC|RULE ported from HOL-Light
Browse files Browse the repository at this point in the history
  • Loading branch information
binghe authored and mn200 committed May 31, 2024
1 parent 7dc35fb commit 77d5e30
Show file tree
Hide file tree
Showing 13 changed files with 1,360 additions and 172 deletions.
20 changes: 15 additions & 5 deletions examples/algebra/ring/Holmakefile
Original file line number Diff line number Diff line change
@@ -1,21 +1,31 @@
INCLUDES = $(HOLDIR)/src/pred_set/src/more_theories $(HOLDIR)/src/integer \
$(HOLDIR)/src/algebra/construction

ifdef POLY
all: $(DEFAULT_TARGETS) selftest.exe
.PHONY: all

HOLHEAP = heap
EXTRA_CLEANS = $(HOLHEAP) selftest.exe ring-selftest.log

selftest.exe: selftest.uo ringLib.uo
$(HOLMOSMLC) -o $@ $<

ifdef POLY
OBJS = pred_set/src/more_theories/cardinalTheory integer/intLib \
algebra/construction/ringTheory

FULL_OBJPATHS = $(patsubst %,$(HOLDIR)/src/%.uo,$(OBJS))

EXTRA_CLEANS = $(HOLHEAP)

all: $(HOLHEAP)

$(HOLHEAP): $(FULL_OBJPATHS) $(HOLDIR)/bin/hol.state
$(protect $(HOLDIR)/bin/buildheap) $(DEBUG_FLAG) -o $@ $(FULL_OBJPATHS)
endif

all: $(DEFAULT_TARGETS)
ifdef HOLSELFTESTLEVEL
all: ring-selftest.log

.PHONY: all
ring-selftest.log: selftest.exe
$(tee ./selftest.exe 2>&1, $@)

endif
15 changes: 15 additions & 0 deletions examples/algebra/ring/ringLib.sig
Original file line number Diff line number Diff line change
@@ -0,0 +1,15 @@
(* ========================================================================= *)
(* A decision procedure for the universal theory of rings *)
(* *)
(* John Harrison, University of Cambridge Computer Laboratory *)
(* (c) Copyright, University of Cambridge 1998 *)
(* ========================================================================= *)

signature ringLib =
sig

include Abbrev

val RING_RULE : term -> thm
val RING_TAC : tactic
end

0 comments on commit 77d5e30

Please sign in to comment.