src/HOL/Import/patches/patch1
author nipkow
Tue, 17 Jun 2025 14:11:40 +0200
changeset 82733 8b537e1af2ec
parent 81931 3c888cd24351
permissions -rw-r--r--
reinstated intersection of lists as inter_list_set
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
81915
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
     1
--- hol-light/statements.ml	1970-01-01 01:00:00.000000000 +0100
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
     2
+++ hol-light-patched/statements.ml	2025-01-18 11:12:11.185279392 +0100
81931
3c888cd24351 discontinue special treatment of HOL Light CONJUNCTS: this is better done in Isabelle;
wenzelm
parents: 81924
diff changeset
     3
@@ -0,0 +1,6 @@
81915
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
     4
+let dump_theorems () =
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
     5
+  let oc = open_out "theorems" in
81931
3c888cd24351 discontinue special treatment of HOL Light CONJUNCTS: this is better done in Isabelle;
wenzelm
parents: 81924
diff changeset
     6
+  output_value oc (map (fun (a,b) -> (a, dest_thm b)) !theorems);
81915
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
     7
+  close_out oc
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
     8
+;;
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
     9
+dump_theorems ();;
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
    10
--- hol-light/stage1.ml	1970-01-01 01:00:00.000000000 +0100
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
    11
+++ hol-light-patched/stage1.ml	2025-01-18 11:12:11.185279392 +0100
81924
61b711122061 allow to load additional HOL Light files, after "hol.ml";
wenzelm
parents: 81919
diff changeset
    12
@@ -0,0 +1,5 @@
81915
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
    13
+#use "hol.ml";;
81924
61b711122061 allow to load additional HOL Light files, after "hol.ml";
wenzelm
parents: 81919
diff changeset
    14
+(*LOAD MORE*)
81915
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
    15
+#use "update_database.ml";;
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
    16
+#use "statements.ml";;
02e107686442 move material from https://gitlab.inria.fr/hol-light-isabelle/hol-light 72b2b702eadb and https://gitlab.inria.fr/hol-light-isabelle/import ce58755b0232 into Isabelle repository: results from running "isabelle component_hol_light_import" of previous version;
wenzelm
parents:
diff changeset
    17
+exit 0;;
81919
f4cd3e679096 clarified patches: avoid duplication;
wenzelm
parents: 81918
diff changeset
    18
--- hol-light/stage2.ml	1970-01-01 01:00:00.000000000 +0100
f4cd3e679096 clarified patches: avoid duplication;
wenzelm
parents: 81918
diff changeset
    19
+++ hol-light-patched/stage2.ml	2025-01-18 11:12:11.384276293 +0100
81924
61b711122061 allow to load additional HOL Light files, after "hol.ml";
wenzelm
parents: 81919
diff changeset
    20
@@ -0,0 +1,4 @@
81919
f4cd3e679096 clarified patches: avoid duplication;
wenzelm
parents: 81918
diff changeset
    21
+#use "hol.ml";;
81924
61b711122061 allow to load additional HOL Light files, after "hol.ml";
wenzelm
parents: 81919
diff changeset
    22
+(*LOAD MORE*)
81919
f4cd3e679096 clarified patches: avoid duplication;
wenzelm
parents: 81918
diff changeset
    23
+stop_recording ();;
f4cd3e679096 clarified patches: avoid duplication;
wenzelm
parents: 81918
diff changeset
    24
+exit 0;;