Skip to content

Commit

Permalink
Merge pull request #574 from binghe/rich_topology
Browse files Browse the repository at this point in the history
hol-light's topology theory and dependents (up to 2015)
  • Loading branch information
Michael Norrish committed Aug 24, 2018
2 parents 83e1331 + f8fd962 commit 6521319
Show file tree
Hide file tree
Showing 11 changed files with 30,327 additions and 606 deletions.
5 changes: 4 additions & 1 deletion src/1/wlogLib.sml
Expand Up @@ -74,7 +74,10 @@ none then "p_hyp" is just "hyp" else it is the splice of "p" with "hyp". The
tuple returned is the aforementioned theorem and "P_hyp". *)
fun wlog_rule vars p hyp t =
let
val the = liteLib.the
(* val the = liteLib.the (broken in mosml) *)
fun the (SOME x) = x
| the _ = failwith "the: can't take \"the\" of NONE"

fun forall vars t = list_mk_forall (vars, t)
fun implies t1 t2 = mk_imp (t1, t2)
val new_sg_t = forall vars (implies (case hyp of
Expand Down
2 changes: 2 additions & 0 deletions src/finite_map/flookupLib.sml
Expand Up @@ -3,6 +3,8 @@ struct

open HolKernel boolLib bossLib finite_mapSyntax

val ERR = mk_HOL_ERR "flookupLib"

(* ------------------------------------------------------------------------- *)

fun memoize size cmp f =
Expand Down
2 changes: 2 additions & 0 deletions src/patricia/patricia_castsSyntax.sml
Expand Up @@ -9,6 +9,8 @@ struct
open Abbrev HolKernel pred_setSyntax wordsSyntax patriciaSyntax
patricia_castsTheory;

val ERR = mk_HOL_ERR "patricia_castsSyntax"

(* ------------------------------------------------------------------------- *)

fun mk_word_ptree_type (aty, bty) =
Expand Down
5 changes: 5 additions & 0 deletions src/pred_set/src/pred_setScript.sml
Expand Up @@ -1363,6 +1363,11 @@ val REST_DEF =
new_definition
("REST_DEF", (“REST (s:'a set) = s DELETE (CHOICE s)”));

val IN_REST = store_thm
("IN_REST",
``!x:'a. !s. x IN (REST s) <=> x IN s /\ ~(x = CHOICE s)``,
REWRITE_TAC [REST_DEF, IN_DELETE]);

val CHOICE_NOT_IN_REST =
store_thm
("CHOICE_NOT_IN_REST",
Expand Down
1,889 changes: 1,889 additions & 0 deletions src/probability/cardScript.sml

Large diffs are not rendered by default.

4,105 changes: 4,105 additions & 0 deletions src/probability/iterateScript.sml

Large diffs are not rendered by default.

607 changes: 607 additions & 0 deletions src/probability/productScript.sml

Large diffs are not rendered by default.

22,765 changes: 22,765 additions & 0 deletions src/probability/rich_topologyScript.sml

Large diffs are not rendered by default.

0 comments on commit 6521319

Please sign in to comment.