Skip to content

Commit

Permalink
A test-case demonstrating the problem with github issue #115.
Browse files Browse the repository at this point in the history
Currently failing so I've put this onto a branch of its own.
  • Loading branch information
mn200 committed Apr 13, 2013
1 parent 4f4b4e2 commit ce19025
Show file tree
Hide file tree
Showing 2 changed files with 29 additions and 0 deletions.
14 changes: 14 additions & 0 deletions src/boss/theory_tests/github115aScript.sml
Original file line number Diff line number Diff line change
@@ -0,0 +1,14 @@
open HolKernel Parse boolLib bossLib

val _ = new_theory "github115a"

open arithmeticTheory

val _ = overload_on ("foo", ``\x. x + y``)

val sample = store_thm(
"sample",
``!y:bool. foo x < foo z ==> x < z``,
SRW_TAC [ARITH_ss][])

val _ = export_theory()
15 changes: 15 additions & 0 deletions src/boss/theory_tests/github115bScript.sml
Original file line number Diff line number Diff line change
@@ -0,0 +1,15 @@
open HolKernel Parse boolLib bossLib

open github115aTheory

(* this theory is in the test-case solely to force Holmake to check that the
github115aTheory.sml file is loadable (it isn't when the bug is evident
because the exception in the execution of export_theory results in a
corrupt Theory.sml file)
*)

val _ = new_theory "github115b"

val sample2 = save_thm("sample2", AND_CLAUSES)

val _ = export_theory()

0 comments on commit ce19025

Please sign in to comment.