lcp [Mon, 14 Nov 1994 10:41:25 +0100] rev 707
Added month for Coens thesis
lcp [Fri, 11 Nov 1994 10:53:41 +0100] rev 706
removal of FOL_dup_cs
lcp [Fri, 11 Nov 1994 10:50:49 +0100] rev 705
removal of HOL_dup_cs
rotation of arguments in split, nat_case, sum_case, list_case
lcp [Fri, 11 Nov 1994 10:42:55 +0100] rev 704
Provers/hypsubst/REPEATN: deleted; using REPEAT_DETERM_N instead.
lcp [Fri, 11 Nov 1994 10:41:09 +0100] rev 703
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
REPEAT_DETERM_SOME: new
lcp [Fri, 11 Nov 1994 10:33:05 +0100] rev 702
FOL/intprover/safe_tac: now uses REPEAT_DETERM_FIRST instead of REPEAT_DETERM
lcp [Fri, 11 Nov 1994 10:31:51 +0100] rev 701
argument swaps in HOL
lcp [Thu, 10 Nov 1994 11:36:40 +0100] rev 700
HOL,ZF/Makefile: enclosed multiple "use" calls in parentheses. This
ensures that if one dies, all die. BUT NOT Pure/Makefile, where
PolyML.use"POLY" makes the identifier "use" visible.
lcp [Thu, 10 Nov 1994 11:06:44 +0100] rev 699
updated pathnames
lcp [Wed, 09 Nov 1994 15:47:11 +0100] rev 698
updated discussion of congruence rules in first section
clasohm [Wed, 09 Nov 1994 13:50:59 +0100] rev 697
changed warning for extremely ambiguous expressions
lcp [Thu, 03 Nov 1994 16:52:19 +0100] rev 696
Pure/goals/prepare_proof/mkresult: now smashes flexflex pairs in the final
result.
lcp [Thu, 03 Nov 1994 16:39:41 +0100] rev 695
ZF/ex/Ramsey,Rmap,misc.ML: modified for new definition of Pi(A,B)
lcp [Thu, 03 Nov 1994 16:05:22 +0100] rev 694
ZF/ex/Ramsey,Rmap,misc.ML: modified for new definition of Pi(A,B)
lcp [Thu, 03 Nov 1994 13:42:39 +0100] rev 693
ZF/Perm/inj_converse_fun: tidied; removed uses of PiI/E
ZF/Perm/comp_fun: tidied; removed use of PiI
lcp [Thu, 03 Nov 1994 12:43:42 +0100] rev 692
ZF/InfDatatype/fun_Vcsucc: removed use of PiE
lcp [Thu, 03 Nov 1994 12:39:39 +0100] rev 691
ZF/func: tidied many proofs, using new definition of Pi(A,B)
ZF/func/PiI,PiE: removed
ZF/func/Pi_iff_old: new
ZF/func/Pi_memberD: new; simpler, replaces memberPiE
lcp [Thu, 03 Nov 1994 12:35:41 +0100] rev 690
ZF: NEW DEFINITION OF PI(A,B)
Was Pi(A,B) == {f: Pow(Sigma(A,B)). ALL x:A. EX! y. <x,y>: f}
Now function(r) == ALL x y. <x,y>:r --> (ALL y'. <x,y'>:r --> y=y')
Pi(A,B) == {f: Pow(Sigma(A,B)). A<=domain(f) & function(f)}"
This simplifies many proofs, since (a) the top-level definition has fewer
bound variables (b) the "total" and "function" properties are separated
(c) the awkward EX! quantifier is eliminated.
ZF/ZF.thy/function: new definition
lcp [Thu, 03 Nov 1994 12:30:55 +0100] rev 689
ZF/Fixedpt/subset_cs: moved to ZF/subset.ML
lcp [Thu, 03 Nov 1994 12:26:59 +0100] rev 688
ZF/Fixedpt/subset0_cs: moved to ZF/ZF.ML
lcp [Thu, 03 Nov 1994 12:23:19 +0100] rev 687
ZF/domrange/converse_iff: new
lcp [Thu, 03 Nov 1994 12:06:37 +0100] rev 686
ZF/upair/theI2: new
lcp [Thu, 03 Nov 1994 11:58:16 +0100] rev 685
ZF/equalities/domain_converse,range_converse,
prod_Un_distrib2,prod_Int_distrib2: new
lcp [Thu, 03 Nov 1994 11:52:04 +0100] rev 684
ZF/Fixedpt/subset0_cs: moved to ZF/ZF.ML
ZF/Fixedpt/subset_cs: moved to ZF/subset.ML
lcp [Thu, 03 Nov 1994 11:45:41 +0100] rev 683
Cardinal_AC/surj_implies_inj: uses Pi_memberD instead of memberPiE
clasohm [Thu, 03 Nov 1994 08:34:53 +0100] rev 682
added warning message
"Currently parsed expression could be extremely ambiguous."
lcp [Wed, 02 Nov 1994 12:48:22 +0100] rev 681
Provers/classical: now takes theorem "classical" as argument, proves "swap"
Provers/classical/depth_tac,deepen_tac: new
lcp [Wed, 02 Nov 1994 12:44:03 +0100] rev 680
Provers/hypsubst: greatly simplified! No longer simulates a
"eres_inst_tac" using rev_cut_eq; instead simply rotates the chosen
equality to the end!
lcp [Wed, 02 Nov 1994 10:45:14 +0100] rev 679
Pure/sign/infer_types/exn_type_msg: new, for more uniform handling of
exception TYPE
nipkow [Wed, 02 Nov 1994 09:09:30 +0100] rev 678
Modified pattern.ML to perform proper matching of Higher-Order Patterns.
Modified thm.ML to preserve bound var names during rewriting.
Renamed eta_matches to matches.
lcp [Tue, 01 Nov 1994 10:40:10 +0100] rev 677
FOL/FOL/swap: deleted
FOL/FOL: tidied the signature
lcp [Tue, 01 Nov 1994 10:32:18 +0100] rev 676
HOLCF/Ssum3.ML: changed res_inst_tac [("P"... to res_inst_tac [("Pa" in
some very ugly proofs. Needed to handle new variable names in swap.
lcp [Mon, 31 Oct 1994 18:15:24 +0100] rev 675
ZF/ZF.thy: added precedences to @RepFun to disambiguate phrases like {x:A.x:B}
lcp [Mon, 31 Oct 1994 18:11:12 +0100] rev 674
ZF/domrange/image_subset: tidied
lcp [Mon, 31 Oct 1994 18:09:32 +0100] rev 673
ZF/upair/mem_asym,succ_inject: tidied
lcp [Mon, 31 Oct 1994 18:07:29 +0100] rev 672
com1,2: added simplifier calls to remove use of ssubst in fast_tac
lcp [Mon, 31 Oct 1994 18:03:14 +0100] rev 671
Pure/tctical/THEN_ELSE: new
lcp [Mon, 31 Oct 1994 18:01:02 +0100] rev 670
Pure/tactic/build_netpair: now takes two arguments
lcp [Mon, 31 Oct 1994 17:59:49 +0100] rev 669
Pure/sequence/hd,tl: new
lcp [Mon, 31 Oct 1994 17:55:43 +0100] rev 668
Pure/drule/thin_rl: new
lcp [Mon, 31 Oct 1994 17:14:42 +0100] rev 667
FOL/ex/ROOT: now loads mini.ML
lcp [Mon, 31 Oct 1994 17:09:10 +0100] rev 666
FOL/ROOT/FOL_dup_cs: removed as obsolete
FOL/ROOT: no longer proves rev_cut_eq for hyp_subst_tac
lcp [Mon, 31 Oct 1994 16:45:19 +0100] rev 665
FOL/ex/cla: proofs now use deepen_tac instead of best_tac FOL_dup_cs
lcp [Mon, 31 Oct 1994 16:39:20 +0100] rev 664
ZF/ZF/ex1_functional: moved to FOL/ROOT
lcp [Mon, 31 Oct 1994 15:49:58 +0100] rev 663
Miniscope conversoin; example of formula rewriting
lcp [Mon, 31 Oct 1994 15:45:54 +0100] rev 662
ZF/OrderArith/thin: deleted as obsolete
ZF/OrderArith/wf_on_radd: now uses thin_rl
lcp [Mon, 31 Oct 1994 15:41:20 +0100] rev 661
added final newline
lcp [Mon, 31 Oct 1994 15:35:43 +0100] rev 660
added header files; deleted commented-out code
nipkow [Fri, 28 Oct 1994 10:13:16 +0100] rev 659
Prepared the code for preservation of bound var names during rewriting. Still
requires a matching function for HO-patterns.
nipkow [Wed, 26 Oct 1994 17:41:40 +0100] rev 658
removed superfluous type_intrs in datatype com.
nipkow [Wed, 26 Oct 1994 15:20:55 +0100] rev 657
simplified syntax of infix continuous functiuons
wenzelm [Tue, 25 Oct 1994 13:16:49 +0100] rev 656
strip_quotes now exported;
wenzelm [Tue, 25 Oct 1994 13:15:34 +0100] rev 655
minor change of occs_const in dest_defn;
wenzelm [Tue, 25 Oct 1994 13:13:52 +0100] rev 654
added require_thy;
lcp [Mon, 24 Oct 1994 10:34:28 +0100] rev 653
HOL,ZF/IMP/Com.thy: tightening precedences to eliminate syntactic ambiguities.
constructor ";" now yields a low precedence; the reduction relations are
now more like infixes.
lcp [Fri, 21 Oct 1994 09:58:05 +0100] rev 652
ZF/intr_elim/elim_rls: now includes Pair_inject, since coinductive
definitions may involve ordinary pairs. (HOL/intr_elim does not require
this change)
lcp [Fri, 21 Oct 1994 09:53:38 +0100] rev 651
Pure/Unify/IMPROVING "CLEANING" OF FLEX-FLEX PAIRS: Old code would refuse
to simplfy %x y.?a(x) =?= %x y.?b(f(?c(y), y)) because it found the flexible
path to y before the rigid path. New code simplifies this to
%x.?a(x) =?= %x.?d, eliminating ?a.
Pure/Unify/rigid_bound: preliminary check for rigid paths to the banned
bound variables
Pure/Unify/change_bnos: any occurrences of the banned bound variables must
now be flexible, causing abandonment of the "cleaning"
lcp [Fri, 21 Oct 1994 09:51:01 +0100] rev 650
LK/hardquant/37: deleted call to flexflex_tac: no longer needed
lcp [Fri, 21 Oct 1994 09:47:02 +0100] rev 649
LCF/LCF.thy: the constant VOID had mixfix syntax "()" !! Added quotes.
lcp [Fri, 21 Oct 1994 09:35:24 +0100] rev 648
FOLP/IFOLP.thy: tightening precedences to eliminate syntactic ambiguities.
Now proof objects have high precedences. Eliminates ambiguity in a=b:P
being parsed as (a=b):P.
lcp [Wed, 19 Oct 1994 09:54:38 +0100] rev 647
ZF/Fixedpt/coinduct: modified proof to suppress deep unification
lcp [Wed, 19 Oct 1994 09:48:13 +0100] rev 646
new comments explaining abandoned change
lcp [Wed, 19 Oct 1994 09:44:31 +0100] rev 645
LCF/fix/lfp_is_FIX: modified proof to suppress deep unification
lcp [Wed, 19 Oct 1994 09:41:48 +0100] rev 644
FOL/ex/cla/58: slightly shorter proof
lcp [Wed, 19 Oct 1994 09:39:23 +0100] rev 643
trivial update to reference
lcp [Wed, 19 Oct 1994 09:23:56 +0100] rev 642
CCL/Gfp/coinduct2, coinduct3: modified proofs to suppress deep unification
CCL/CCL, Fix, Gfp, Hered, Set, Term, Trancl, Type, Wfd: expanded shorthands
wenzelm [Wed, 12 Oct 1994 16:38:58 +0100] rev 641
add_defs: improved error messages;
installed new print_goals with nice 'env mode';
wenzelm [Wed, 12 Oct 1994 16:34:52 +0100] rev 640
removed old comment;
wenzelm [Wed, 12 Oct 1994 16:34:00 +0100] rev 639
remove _explode, _implode and trfuns;
wenzelm [Wed, 12 Oct 1994 16:32:06 +0100] rev 638
prove_subclass, prove_arity now exported;
minor internal changes;
wenzelm [Wed, 12 Oct 1994 16:31:01 +0100] rev 637
added is_equals: term -> bool;
wenzelm [Wed, 12 Oct 1994 16:30:19 +0100] rev 636
type_args, opt_witness now exported;
added AxClass.;
wenzelm [Wed, 12 Oct 1994 16:29:10 +0100] rev 635
AxClass no longer open;
lcp [Wed, 12 Oct 1994 12:20:18 +0100] rev 634
{HOL,ZF}/intr_elim/intro_tacsf: now calls DEPTH_SOLVE_1 instead of REPEAT to
solve the goal fully
lcp [Wed, 12 Oct 1994 12:09:54 +0100] rev 633
{HOL,ZF}/indrule/ind_tac: now calls DEPTH_SOLVE_1 instead of REPEAT, to
solve the goal fully before proceeding
{HOL,ZF}/indrule/mutual_ind_tac: ensures that calls to "prem" cannot loop;
calls DEPTH_SOLVE_1 instead of REPEAT to solve the goal fully
wenzelm [Wed, 12 Oct 1994 11:09:11 +0100] rev 632
fixed infix names in print_translations;
lcp [Wed, 12 Oct 1994 09:48:32 +0100] rev 631
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
next tactical call. There is no good way of doing this because of
backtracking.
Pure/tctical/exec_trace_command,tracify,traced_tac: these set, test and
reset suppress_tracing
lcp [Wed, 12 Oct 1994 09:42:32 +0100] rev 630
Minor reference updates
lcp [Wed, 12 Oct 1994 09:20:17 +0100] rev 629
Moving theory LList to ex directory
nipkow [Mon, 10 Oct 1994 18:09:58 +0100] rev 628
corrected problems with changed binding power of ::.
nipkow [Mon, 10 Oct 1994 12:57:23 +0100] rev 627
README file
clasohm [Sat, 08 Oct 1994 13:45:40 +0100] rev 626
changed precedences of _constrain (i.e. "::")
nipkow [Thu, 06 Oct 1994 18:40:18 +0100] rev 625
New version
clasohm [Tue, 04 Oct 1994 13:02:16 +0100] rev 624
made major changes to grammar;
added call of Type.infer_types to automatically eliminate ambiguities
clasohm [Tue, 04 Oct 1994 13:01:17 +0100] rev 623
added print_msg;
added call of Type.infer_types to resolve ambiguities
nipkow [Tue, 27 Sep 1994 14:23:46 +0100] rev 622
Modified termord to take account of the Abs-Abs case.
wenzelm [Mon, 26 Sep 1994 17:56:21 +0100] rev 621
improved expand_typ (now handles TVars);
slightly changed ext_tsig_abbrs;
added ext_tsig_arities;
removed extend_tsig;
various internal changes;
wenzelm [Mon, 26 Sep 1994 17:55:45 +0100] rev 620
exported pretty_sort;
various minor internal changes;
wenzelm [Mon, 26 Sep 1994 17:36:10 +0100] rev 619
added init_pps;
wenzelm [Mon, 26 Sep 1994 17:35:45 +0100] rev 618
added init_database (somewhat experimental);
wenzelm [Mon, 26 Sep 1994 17:35:23 +0100] rev 617
added flag show_no_free_types: bool ref;
wenzelm [Mon, 26 Sep 1994 17:34:59 +0100] rev 616
explode_tr now produces leadings 0s;
implode_ast_tr' now quotes result;
wenzelm [Wed, 21 Sep 1994 15:39:02 +0200] rev 615
minor cleanup, added 'syntax' section;
lcp [Thu, 15 Sep 1994 13:13:54 +0200] rev 614
now mentions that the sections are available as
Datatypes and (Co)Inductive Definitions in Isabelle/HOL
wenzelm [Wed, 14 Sep 1994 16:11:19 +0200] rev 613
removed lookup_const (use Sign.const_type instead);
wenzelm [Wed, 14 Sep 1994 16:05:39 +0200] rev 612
replaced lookup_const by Sign.const_type;
wenzelm [Wed, 14 Sep 1994 16:02:06 +0200] rev 611
now uses Sign.const_type;
wenzelm [Wed, 14 Sep 1994 14:49:56 +0200] rev 610
letrec syntax: replaced "id" by "idt";
lcp [Tue, 13 Sep 1994 11:39:49 +0200] rev 609
updated for Isabelle94
lcp [Tue, 13 Sep 1994 11:19:38 +0200] rev 608
now uses find to locate .thy.ML files everywhere
lcp [Tue, 13 Sep 1994 10:42:34 +0200] rev 607
updated the identifier "version"
lcp [Tue, 13 Sep 1994 10:26:24 +0200] rev 606
minor updates
lcp [Mon, 12 Sep 1994 13:20:07 +0200] rev 605
New Makefile for Logics Manual
lcp [Mon, 12 Sep 1994 13:06:07 +0200] rev 604
New Makefile for Reference Manual
lcp [Mon, 12 Sep 1994 13:01:38 +0200] rev 603
New Makefile for Introduction
lcp [Mon, 12 Sep 1994 12:45:10 +0200] rev 602
New Makefile for ind-defs
nipkow [Sun, 11 Sep 1994 12:52:00 +0200] rev 601
Added primrec section
nipkow [Sun, 11 Sep 1994 10:59:09 +0200] rev 600
Added primrec section.
lcp [Fri, 09 Sep 1994 13:10:09 +0200] rev 599
now in a format that could be published
lcp [Fri, 09 Sep 1994 12:34:54 +0200] rev 598
added Abrial and Laffitte; Kunen; Winskel, etc.
lcp [Fri, 09 Sep 1994 12:25:56 +0200] rev 597
Updated for existence of HOL version and infinitely
branching datatypes
lcp [Fri, 09 Sep 1994 11:57:49 +0200] rev 596
Per cent (%) now functions as comment character in tt
box environment
lcp [Fri, 09 Sep 1994 11:52:38 +0200] rev 595
Added mention of directory IMP; tidied the section on examples.
lcp [Fri, 09 Sep 1994 11:45:44 +0200] rev 594
Logics/HOL: Section 3, added Pow and its rule. New sections 6 on the
datatype declaration and 7 on (co)inductive definitions. Added mention of
directory IMP.
lcp [Fri, 09 Sep 1994 11:40:40 +0200] rev 593
ZF/Zorn/next_bounded: deleted this proof, which was already in comments
lcp [Thu, 08 Sep 1994 13:17:57 +0200] rev 592
documentation on theories
lcp [Thu, 08 Sep 1994 12:55:50 +0200] rev 591
ZF/add_ind_def/add_fp_def_i: now prints the fixedpoint defs at the terminal
lcp [Thu, 08 Sep 1994 11:05:06 +0200] rev 590
{HOL,ZF}/indrule/quant_induct: replaced ssubst in eresolve_tac by
separate call to hyp_subst_tac. This avoids substituting in x=f(x)
{HOL,ZF}/indrule/ind_tac: now tries resolve_tac [refl]. This handles
trivial equalities such as x=a.
{HOL,ZF}/intr_elim/intro_tacsf_tac: now calls assume_tac last, to try refl
before any equality assumptions
lcp [Wed, 07 Sep 1994 17:28:53 +0200] rev 589
addition of ZF/ex/twos_compl.thy
clasohm [Wed, 07 Sep 1994 13:04:28 +0200] rev 588
moved from Contrib
clasohm [Wed, 07 Sep 1994 10:43:30 +0200] rev 587
renamed temporary variable 'base' to 'thy' in mk_structure
clasohm [Tue, 06 Sep 1994 14:44:10 +0200] rev 586
renamed base_on into mk_base and moved it to the beginning of the generated
.thy.ML file to make sure that all base theories are present when ML executes
the rest of this file
lcp [Tue, 06 Sep 1994 13:46:53 +0200] rev 585
Pure/type/unvarifyT: moved there from logic.ML
lcp [Tue, 06 Sep 1994 13:28:56 +0200] rev 584
documentation of theory sections (co)inductive and (co)datatype
wenzelm [Tue, 06 Sep 1994 13:10:38 +0200] rev 583
minor internal changes;
wenzelm [Tue, 06 Sep 1994 13:09:58 +0200] rev 582
added ext_tsig_types;
various minor changes;
lcp [Tue, 06 Sep 1994 11:02:16 +0200] rev 581
removal of needless quotes
nipkow [Wed, 31 Aug 1994 17:34:12 +0200] rev 580
Updated datatype documentation with a few hints
lcp [Thu, 25 Aug 1994 12:21:00 +0200] rev 579
new file of useful things for writing theory sections
lcp [Thu, 25 Aug 1994 12:09:21 +0200] rev 578
ZF/Inductive.thy,.ML: renamed from "inductive" to allow re-building without
the keyword "inductive" making the theory file fail
ZF/Makefile: now has Inductive.thy,.ML
ZF/Datatype,Finite,Zorn: depend upon Inductive
ZF/intr_elim: now checks that the inductive name does not clash with
existing theory names
ZF/ind_section: deleted things replicated in Pure/section_utils.ML
ZF/ROOT: now loads Pure/section_utils
lcp [Thu, 25 Aug 1994 10:41:17 +0200] rev 577
print_sign_exn: now exported, with a polymorphic type
lcp [Wed, 24 Aug 1994 15:48:47 +0200] rev 576
ZF/ex/LList/lconst_type: streamlined proof
wenzelm [Tue, 23 Aug 1994 19:34:01 +0200] rev 575
added print_syntax: theory -> unit;
wenzelm [Tue, 23 Aug 1994 19:33:33 +0200] rev 574
read_def_cterm: minor changes;
merge_thm_sgs: improved error msg;
wenzelm [Tue, 23 Aug 1994 19:31:05 +0200] rev 573
removed constant _constrain from Pure sig;
lcp [Mon, 22 Aug 1994 11:27:23 +0200] rev 572
ZF/upair/consE', UnE': new
lcp [Mon, 22 Aug 1994 11:11:17 +0200] rev 571
ZF/Cardinal: some results moved here from CardinalArith
ZF/CardinalArith/nat_succ_lepoll: removed obsolete proof
ZF/CardinalArith/nat_cons_eqpoll: new
lcp [Mon, 22 Aug 1994 11:07:40 +0200] rev 570
Pure/Thy/thy_parse/THY_PARSE: deleted duplicate specifications of parens,
brackets, ..., mk_triple
lcp [Mon, 22 Aug 1994 11:03:52 +0200] rev 569
HOLCF/Lift1.thy: now imports Sum
wenzelm [Fri, 19 Aug 1994 16:13:53 +0200] rev 568
replaced Lexicon.scan_id by Scanner.scan_id;
replaced const_name by Syntax.const_name;
wenzelm [Fri, 19 Aug 1994 16:12:23 +0200] rev 567
replaced add_defns_i by add_defs_i;
wenzelm [Fri, 19 Aug 1994 16:09:27 +0200] rev 566
replaced sextension.ML by syn_trans.ML;
wenzelm [Fri, 19 Aug 1994 15:42:13 +0200] rev 565
slightly changed args of infer_types;
replaced parents by enclose;
renamed 2nd add_types to attach_types and fixed the
typevar-sort-constraint BUG;
various minor internal changes;
wenzelm [Fri, 19 Aug 1994 15:41:39 +0200] rev 564
added inferT_axm;
removed extend_theory;
changed read_def_cterm: now uses Sign.infer_types;
wenzelm [Fri, 19 Aug 1994 15:41:00 +0200] rev 563
replaced mapst by map;
added find_first;
wenzelm [Fri, 19 Aug 1994 15:40:44 +0200] rev 562
added pretty_sg;
added infer_types;
removed subclasses arg of add_classes;
removed old 'extend' and related stuff;
various minor internal changes;
wenzelm [Fri, 19 Aug 1994 15:40:10 +0200] rev 561
added add_defs, add_defs_i;
wenzelm [Fri, 19 Aug 1994 15:39:52 +0200] rev 560
cleaned sig;
removed add_defns (now in drule.ML as add_defs);
removed add_sigclass;
minor internal changes;
wenzelm [Fri, 19 Aug 1994 15:39:19 +0200] rev 559
added theory_of_sign, theory_of_thm;
renamed get_thms to thms_of;
improved store_thms etc.;
wenzelm [Fri, 19 Aug 1994 15:38:50 +0200] rev 558
renamed 'defns' to 'defs';
removed 'sigclass';
replaced parents by enclose;
exported parens, brackets, mk_list, mk_big_list, mk_pair, mk_triple;
various minor internal changes;
wenzelm [Fri, 19 Aug 1994 15:38:18 +0200] rev 557
added raw_term_sorts and changed typ_of_term accordingly (part of fix
of the typevar-sort-constraint BUG);
various minor internal changes;
wenzelm [Fri, 19 Aug 1994 15:37:46 +0200] rev 556
added type xrule (from sextension.ML);
removed old 'extend';
removed added syn_ext_const_names, syn_ext_trfuns (now in syn_ext.ML);
various minor changes;
wenzelm [Fri, 19 Aug 1994 15:37:24 +0200] rev 555
removed idT, varT, tidT, tvarT (now in lexicon.ML);
added syn_ext_const_names, syn_ext_trfuns;
wenzelm [Fri, 19 Aug 1994 15:37:05 +0200] rev 554
various minor internal changes;
wenzelm [Fri, 19 Aug 1994 15:36:45 +0200] rev 553
added map_strs: (string -> string) -> T -> T;
wenzelm [Fri, 19 Aug 1994 15:36:23 +0200] rev 552
removed roots arg of extend_gram;
added functor sig constraint (: PARSER);
wenzelm [Fri, 19 Aug 1994 15:35:56 +0200] rev 551
minor cleanings;
wenzelm [Fri, 19 Aug 1994 15:35:38 +0200] rev 550
replaced id, var, tid, tvar by idT, varT, tidT, tvarT;
added const, free, var: build atomic terms of dummyT;
added 'xnum' (signed numerals) and 'xstr' (strings) token kinds;
various minor internal changes;
wenzelm [Fri, 19 Aug 1994 15:34:58 +0200] rev 549
replaced SExtension by SynTrans (mixfix stuff in Mixfix);
private structs now hidden within PrivateSyntax;
wenzelm [Fri, 19 Aug 1994 15:34:28 +0200] rev 548
added this file;
lcp [Fri, 19 Aug 1994 10:57:40 +0200] rev 547
deleted obsolete references to ISABELLEMAKE
lcp [Thu, 18 Aug 1994 17:56:07 +0200] rev 546
/unvarifyT, unvarify: moved to Pure/logic.ML
lcp [Thu, 18 Aug 1994 17:53:28 +0200] rev 545
Pure/goals.ML: prove_goalw_cterm now does its own exception-handling, moved
from prove_goalw
lcp [Thu, 18 Aug 1994 17:50:22 +0200] rev 544
Pure/library/assert_all: new, moved from ZF/ind_syntax.ML
lcp [Thu, 18 Aug 1994 17:41:40 +0200] rev 543
ZF/ind_syntax/unvarifyT, unvarify: moved to Pure/logic.ML
ZF/ind_syntax/prove_term: deleted
ZF/constructor, indrule, intr_elim: now call prove_goalw_cterm and
Logic.unvarify
lcp [Thu, 18 Aug 1994 12:56:57 +0200] rev 542
HOLCF/Lift1.thy: updated for new sum_case by using "case" syntax
lcp [Wed, 17 Aug 1994 10:42:41 +0200] rev 541
overheads for inductive definitions, originally for CADE-12
lcp [Wed, 17 Aug 1994 10:38:37 +0200] rev 540
ZF/ex/ROOT: added .ML to use command use "ex/twos_compl"
Should be able to delete this after fixing the treatment of orphans.
lcp [Wed, 17 Aug 1994 10:34:44 +0200] rev 539
ZF/ex/Ntree: two new examples, maptree and maptree2
lcp [Wed, 17 Aug 1994 10:33:23 +0200] rev 538
ZF/func/fun_extend3: new
ZF/func/cons_fun_eq: simplified proof
lcp [Wed, 17 Aug 1994 10:31:35 +0200] rev 537
ZF/Univ/Sigma_subset_univ, Transset_Pair_subset_univ: deleted
lcp [Tue, 16 Aug 1994 19:09:43 +0200] rev 536
ZF/domrange/domain_of_prod, domain_empty, etc: moved to equalities.ML where
they can be proved trivially using eq_cs
ZF/domrange/XXX_empty: renamed XXX_0
lcp [Tue, 16 Aug 1994 19:06:14 +0200] rev 535
ZF/ex/Equiv.thy,.ML: moved to main directory as EquivClass.thy,.ML
lcp [Tue, 16 Aug 1994 19:03:45 +0200] rev 534
ZF/Finite: added the finite function space, A-||>B
ZF/InfDatatype: added rules for the above
lcp [Tue, 16 Aug 1994 19:01:26 +0200] rev 533
ZF/pair.ML: moved some definitions here from simpdata.ML
lcp [Tue, 16 Aug 1994 18:58:42 +0200] rev 532
ZF/Makefile,ROOT.ML, ZF/ex/Integ.thy: updated for EquivClass
lcp [Tue, 16 Aug 1994 18:53:29 +0200] rev 531
ZF/Makefile,ROOT.ML, ZF/ex/Integ.thy: updated for EquivClass
lcp [Mon, 15 Aug 1994 19:01:51 +0200] rev 530
ZF/Makefile/FILES: added many missing .thy files
lcp [Mon, 15 Aug 1994 18:38:38 +0200] rev 529
ZF/List, ex/Brouwer,Data,LList,Ntree,TF,Term: much simplified proof of _unfold
lcp [Mon, 15 Aug 1994 18:37:25 +0200] rev 528
ZF/ex/Brouwer.thy,.ML: new example of wellordering types
lcp [Mon, 15 Aug 1994 18:31:29 +0200] rev 527
ZF/ex/CoUnit/lleq_cs: copied from LList.ML
lcp [Mon, 15 Aug 1994 18:27:50 +0200] rev 526
ZF/ex/ROOT: changed "time_use" to "time_use_thy" to load CoUnit;
removed some explicit loads by exploiting theory dependencies
lcp [Mon, 15 Aug 1994 18:25:27 +0200] rev 525
ZF/List, ex/Brouwer,Data,LList,Ntree,TF,Term: much simplified proof of _unfold
lcp [Mon, 15 Aug 1994 18:15:09 +0200] rev 524
ZF/InfDatatype: simplified, extended results for infinite branching
lcp [Mon, 15 Aug 1994 18:12:56 +0200] rev 523
ZF/CardinalArith/InfCard_Un: new
lcp [Mon, 15 Aug 1994 18:11:00 +0200] rev 522
ZF/Cardinal/Card_Un: new
lcp [Mon, 15 Aug 1994 18:09:37 +0200] rev 521
ZF/Sum/Sigma_bool: new
lcp [Mon, 15 Aug 1994 18:07:03 +0200] rev 520
ZF/equalities/Sigma_cons: new
ZF/equalities/cons_eq: new
ZF/equalities.thy: added final newline
lcp [Mon, 15 Aug 1994 18:04:10 +0200] rev 519
ZF/func/empty_fun: renamed from fun_empty
ZF/func/single_fun: replaces the weaker fun_single
ZF/func/fun_single_lemma: deleted
ZF/func.thy: now depends upon equalities.thy
nipkow [Mon, 15 Aug 1994 16:12:35 +0200] rev 518
Proof beautification
lcp [Fri, 12 Aug 1994 18:45:33 +0200] rev 517
for infinite datatypes with arbitrary index sets
lcp [Fri, 12 Aug 1994 12:51:34 +0200] rev 516
installation of new inductive/datatype sections
lcp [Fri, 12 Aug 1994 12:28:46 +0200] rev 515
installation of new inductive/datatype sections
lcp [Fri, 12 Aug 1994 11:13:23 +0200] rev 514
addition of string escapes
lcp [Fri, 12 Aug 1994 11:01:18 +0200] rev 513
updated reference to parents
lcp [Fri, 12 Aug 1994 10:57:55 +0200] rev 512
Pure/library/enclose, Pure/Syntax/pretty/enclose: renamed from parents
Pure/library/is_blank: now handles form feeds () too, in accordance with
ML definition
lcp [Fri, 12 Aug 1994 10:20:07 +0200] rev 511
re-organized using new theory sections
nipkow [Mon, 08 Aug 1994 16:45:08 +0200] rev 510
Simplified some proofs. Added some type assumptions to the introduction rules.
lcp [Thu, 04 Aug 1994 12:39:28 +0200] rev 509
fixed spelling
lcp [Thu, 04 Aug 1994 11:51:30 +0200] rev 508
addition of show_brackets
lcp [Thu, 04 Aug 1994 11:45:59 +0200] rev 507
addition of show_brackets
nipkow [Wed, 03 Aug 1994 09:45:42 +0200] rev 506
improved show_brackets again - Trueprop does not create () any more.
nipkow [Tue, 02 Aug 1994 20:08:57 +0200] rev 505
minimized () in forced printing of barckets (show_brackets)
nipkow [Tue, 02 Aug 1994 09:07:10 +0200] rev 504
added flag show_brackets for printinmg fully bracketed terms.
lcp [Mon, 01 Aug 1994 17:34:57 +0200] rev 503
trivial whitespace change
lcp [Mon, 01 Aug 1994 17:24:46 +0200] rev 502
ZF/Perm.ML/inj_converse_inj, comp_inj: simpler proofs using f_imp_injective
many other tidies
lcp [Fri, 29 Jul 1994 16:07:22 +0200] rev 501
ZF/ex/PropLog/sat_XXX: renamed logcon_XXX, since the relation is logical
consequence rather than satisfaction
nipkow [Fri, 29 Jul 1994 15:32:17 +0200] rev 500
some small simplifications
lcp [Fri, 29 Jul 1994 13:30:48 +0200] rev 499
deleted repeated "the" in "before the the .thy file"
lcp [Fri, 29 Jul 1994 13:28:39 +0200] rev 498
renamed union_iff to Union_iff
renamed power_set to Pow_iff
DiffD2: now is really a destruction rule
lcp [Fri, 29 Jul 1994 13:21:26 +0200] rev 497
revised for new theory system: removal of ext, addition of thy_name
lcp [Fri, 29 Jul 1994 11:09:45 +0200] rev 496
Inductive defs need no longer mention SigmaI/E2
lcp [Fri, 29 Jul 1994 11:03:23 +0200] rev 495
ZF/intr_elim/intro_tacsf: now uses SigmaI as a default intro rule and
SigmaE2 as a default elim rule
lcp [Thu, 28 Jul 1994 12:44:40 +0200] rev 494
ZF/WF/wf_induct: streamlined proof
lcp [Thu, 28 Jul 1994 11:25:37 +0200] rev 493
ZF/constructor.thy: now specifies intr_elim as its parent; previously had
ind_syntax, which was not sufficient.
lcp [Wed, 27 Jul 1994 19:08:14 +0200] rev 492
added a new example due to Robin Arthan
lcp [Wed, 27 Jul 1994 19:04:21 +0200] rev 491
logics update
lcp [Wed, 27 Jul 1994 16:09:14 +0200] rev 490
Addition of infinite branching datatypes
lcp [Wed, 27 Jul 1994 16:03:16 +0200] rev 489
Addition of infinite branching datatypes
lcp [Wed, 27 Jul 1994 15:33:42 +0200] rev 488
Addition of infinite branching datatypes
wenzelm [Wed, 27 Jul 1994 15:14:31 +0200] rev 487
added experimental add_defns (actually should be moved somewhere else);
minor internal changes;
lcp [Tue, 26 Jul 1994 14:02:16 +0200] rev 486
Misc minor updates
lcp [Tue, 26 Jul 1994 13:44:42 +0200] rev 485
Axiom of choice, cardinality results, etc.
lcp [Tue, 26 Jul 1994 13:21:20 +0200] rev 484
Axiom of choice, cardinality results, etc.
nipkow [Thu, 21 Jul 1994 16:51:26 +0200] rev 483
added IMP
nipkow [Thu, 21 Jul 1994 14:27:00 +0200] rev 482
Initial revision
nipkow [Thu, 21 Jul 1994 14:05:34 +0200] rev 481
Initial revision
wenzelm [Wed, 20 Jul 1994 12:09:48 +0200] rev 480
fixed comment: "(| _ : _ |)" to "OFCLASS(_, _)"
nipkow [Mon, 18 Jul 1994 12:24:35 +0200] rev 479
*** empty log message ***
nipkow [Mon, 18 Jul 1994 12:22:30 +0200] rev 478
added init_thy_reader and removed extend_theory
clasohm [Fri, 15 Jul 1994 13:34:31 +0200] rev 477
added thy_name to Datatype_Fun's parameter
clasohm [Fri, 15 Jul 1994 13:30:42 +0200] rev 476
added check for concistency of filename and theory name;
made loaded_thys a symtab instead of an association list;
added store_thm, qed, get_thm, get_thms
clasohm [Fri, 15 Jul 1994 12:24:05 +0200] rev 475
added function mapst
wenzelm [Thu, 14 Jul 1994 11:39:25 +0200] rev 474
added functor signature constraint;
wenzelm [Thu, 14 Jul 1994 11:38:24 +0200] rev 473
minor internal renamings;
wenzelm [Thu, 14 Jul 1994 11:37:08 +0200] rev 472
changed syntax "(| _ : _ |)" to "OFCLASS(_, _)";
lcp [Wed, 13 Jul 1994 10:13:52 +0200] rev 471
indentation and renaming of rules
lcp [Tue, 12 Jul 1994 18:38:39 +0200] rev 470
minor updates
lcp [Tue, 12 Jul 1994 18:30:53 +0200] rev 469
chain_tac: deleted; just use etac mp
lcp [Tue, 12 Jul 1994 18:20:39 +0200] rev 468
Improved error checking