Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-480
+480
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
replaced lookup_const by Sign.const_type;
1994-09-14, by wenzelm
now uses Sign.const_type;
1994-09-14, by wenzelm
letrec syntax: replaced "id" by "idt";
1994-09-14, by wenzelm
updated for Isabelle94
1994-09-13, by lcp
now uses find to locate .thy.ML files everywhere
1994-09-13, by lcp
updated the identifier "version"
1994-09-13, by lcp
minor updates
1994-09-13, by lcp
New Makefile for Logics Manual
1994-09-12, by lcp
New Makefile for Reference Manual
1994-09-12, by lcp
New Makefile for Introduction
1994-09-12, by lcp
New Makefile for ind-defs
1994-09-12, by lcp
Added primrec section
1994-09-11, by nipkow
Added primrec section.
1994-09-11, by nipkow
now in a format that could be published
1994-09-09, by lcp
added Abrial and Laffitte; Kunen; Winskel, etc.
1994-09-09, by lcp
Updated for existence of HOL version and infinitely
1994-09-09, by lcp
Per cent (%) now functions as comment character in tt
1994-09-09, by lcp
Added mention of directory IMP; tidied the section on examples.
1994-09-09, by lcp
Logics/HOL: Section 3, added Pow and its rule. New sections 6 on the
1994-09-09, by lcp
ZF/Zorn/next_bounded: deleted this proof, which was already in comments
1994-09-09, by lcp
documentation on theories
1994-09-08, by lcp
ZF/add_ind_def/add_fp_def_i: now prints the fixedpoint defs at the terminal
1994-09-08, by lcp
{HOL,ZF}/indrule/quant_induct: replaced ssubst in eresolve_tac by
1994-09-08, by lcp
addition of ZF/ex/twos_compl.thy
1994-09-07, by lcp
moved from Contrib
1994-09-07, by clasohm
renamed temporary variable 'base' to 'thy' in mk_structure
1994-09-07, by clasohm
renamed base_on into mk_base and moved it to the beginning of the generated
1994-09-06, by clasohm
Pure/type/unvarifyT: moved there from logic.ML
1994-09-06, by lcp
documentation of theory sections (co)inductive and (co)datatype
1994-09-06, by lcp
minor internal changes;
1994-09-06, by wenzelm
added ext_tsig_types;
1994-09-06, by wenzelm
removal of needless quotes
1994-09-06, by lcp
Updated datatype documentation with a few hints
1994-08-31, by nipkow
new file of useful things for writing theory sections
1994-08-25, by lcp
ZF/Inductive.thy,.ML: renamed from "inductive" to allow re-building without
1994-08-25, by lcp
print_sign_exn: now exported, with a polymorphic type
1994-08-25, by lcp
ZF/ex/LList/lconst_type: streamlined proof
1994-08-24, by lcp
added print_syntax: theory -> unit;
1994-08-23, by wenzelm
read_def_cterm: minor changes;
1994-08-23, by wenzelm
removed constant _constrain from Pure sig;
1994-08-23, by wenzelm
ZF/upair/consE', UnE': new
1994-08-22, by lcp
ZF/Cardinal: some results moved here from CardinalArith
1994-08-22, by lcp
Pure/Thy/thy_parse/THY_PARSE: deleted duplicate specifications of parens,
1994-08-22, by lcp
HOLCF/Lift1.thy: now imports Sum
1994-08-22, by lcp
replaced Lexicon.scan_id by Scanner.scan_id;
1994-08-19, by wenzelm
replaced add_defns_i by add_defs_i;
1994-08-19, by wenzelm
replaced sextension.ML by syn_trans.ML;
1994-08-19, by wenzelm
slightly changed args of infer_types;
1994-08-19, by wenzelm
added inferT_axm;
1994-08-19, by wenzelm
replaced mapst by map;
1994-08-19, by wenzelm
added pretty_sg;
1994-08-19, by wenzelm
added add_defs, add_defs_i;
1994-08-19, by wenzelm
cleaned sig;
1994-08-19, by wenzelm
added theory_of_sign, theory_of_thm;
1994-08-19, by wenzelm
renamed 'defns' to 'defs';
1994-08-19, by wenzelm
added raw_term_sorts and changed typ_of_term accordingly (part of fix
1994-08-19, by wenzelm
added type xrule (from sextension.ML);
1994-08-19, by wenzelm
removed idT, varT, tidT, tvarT (now in lexicon.ML);
1994-08-19, by wenzelm
various minor internal changes;
1994-08-19, by wenzelm
added map_strs: (string -> string) -> T -> T;
1994-08-19, by wenzelm
removed roots arg of extend_gram;
1994-08-19, by wenzelm
minor cleanings;
1994-08-19, by wenzelm
replaced id, var, tid, tvar by idT, varT, tidT, tvarT;
1994-08-19, by wenzelm
replaced SExtension by SynTrans (mixfix stuff in Mixfix);
1994-08-19, by wenzelm
added this file;
1994-08-19, by wenzelm
deleted obsolete references to ISABELLEMAKE
1994-08-19, by lcp
/unvarifyT, unvarify: moved to Pure/logic.ML
1994-08-18, by lcp
Pure/goals.ML: prove_goalw_cterm now does its own exception-handling, moved
1994-08-18, by lcp
Pure/library/assert_all: new, moved from ZF/ind_syntax.ML
1994-08-18, by lcp
ZF/ind_syntax/unvarifyT, unvarify: moved to Pure/logic.ML
1994-08-18, by lcp
HOLCF/Lift1.thy: updated for new sum_case by using "case" syntax
1994-08-18, by lcp
overheads for inductive definitions, originally for CADE-12
1994-08-17, by lcp
ZF/ex/ROOT: added .ML to use command use "ex/twos_compl"
1994-08-17, by lcp
ZF/ex/Ntree: two new examples, maptree and maptree2
1994-08-17, by lcp
ZF/func/fun_extend3: new
1994-08-17, by lcp
ZF/Univ/Sigma_subset_univ, Transset_Pair_subset_univ: deleted
1994-08-17, by lcp
ZF/domrange/domain_of_prod, domain_empty, etc: moved to equalities.ML where
1994-08-16, by lcp
ZF/ex/Equiv.thy,.ML: moved to main directory as EquivClass.thy,.ML
1994-08-16, by lcp
ZF/Finite: added the finite function space, A-||>B
1994-08-16, by lcp
ZF/pair.ML: moved some definitions here from simpdata.ML
1994-08-16, by lcp
ZF/Makefile,ROOT.ML, ZF/ex/Integ.thy: updated for EquivClass
1994-08-16, by lcp
ZF/Makefile,ROOT.ML, ZF/ex/Integ.thy: updated for EquivClass
1994-08-16, by lcp
ZF/Makefile/FILES: added many missing .thy files
1994-08-15, by lcp
ZF/List, ex/Brouwer,Data,LList,Ntree,TF,Term: much simplified proof of _unfold
1994-08-15, by lcp
ZF/ex/Brouwer.thy,.ML: new example of wellordering types
1994-08-15, by lcp
ZF/ex/CoUnit/lleq_cs: copied from LList.ML
1994-08-15, by lcp
ZF/ex/ROOT: changed "time_use" to "time_use_thy" to load CoUnit;
1994-08-15, by lcp
ZF/List, ex/Brouwer,Data,LList,Ntree,TF,Term: much simplified proof of _unfold
1994-08-15, by lcp
ZF/InfDatatype: simplified, extended results for infinite branching
1994-08-15, by lcp
ZF/CardinalArith/InfCard_Un: new
1994-08-15, by lcp
ZF/Cardinal/Card_Un: new
1994-08-15, by lcp
ZF/Sum/Sigma_bool: new
1994-08-15, by lcp
ZF/equalities/Sigma_cons: new
1994-08-15, by lcp
ZF/func/empty_fun: renamed from fun_empty
1994-08-15, by lcp
Proof beautification
1994-08-15, by nipkow
for infinite datatypes with arbitrary index sets
1994-08-12, by lcp
installation of new inductive/datatype sections
1994-08-12, by lcp
installation of new inductive/datatype sections
1994-08-12, by lcp
addition of string escapes
1994-08-12, by lcp
updated reference to parents
1994-08-12, by lcp
Pure/library/enclose, Pure/Syntax/pretty/enclose: renamed from parents
1994-08-12, by lcp
re-organized using new theory sections
1994-08-12, by lcp
Simplified some proofs. Added some type assumptions to the introduction rules.
1994-08-08, by nipkow
fixed spelling
1994-08-04, by lcp
addition of show_brackets
1994-08-04, by lcp
addition of show_brackets
1994-08-04, by lcp
improved show_brackets again - Trueprop does not create () any more.
1994-08-03, by nipkow
minimized () in forced printing of barckets (show_brackets)
1994-08-02, by nipkow
added flag show_brackets for printinmg fully bracketed terms.
1994-08-02, by nipkow
trivial whitespace change
1994-08-01, by lcp
ZF/Perm.ML/inj_converse_inj, comp_inj: simpler proofs using f_imp_injective
1994-08-01, by lcp
ZF/ex/PropLog/sat_XXX: renamed logcon_XXX, since the relation is logical
1994-07-29, by lcp
some small simplifications
1994-07-29, by nipkow
deleted repeated "the" in "before the the .thy file"
1994-07-29, by lcp
renamed union_iff to Union_iff
1994-07-29, by lcp
revised for new theory system: removal of ext, addition of thy_name
1994-07-29, by lcp
Inductive defs need no longer mention SigmaI/E2
1994-07-29, by lcp
ZF/intr_elim/intro_tacsf: now uses SigmaI as a default intro rule and
1994-07-29, by lcp
ZF/WF/wf_induct: streamlined proof
1994-07-28, by lcp
ZF/constructor.thy: now specifies intr_elim as its parent; previously had
1994-07-28, by lcp
added a new example due to Robin Arthan
1994-07-27, by lcp
logics update
1994-07-27, by lcp
Addition of infinite branching datatypes
1994-07-27, by lcp
Addition of infinite branching datatypes
1994-07-27, by lcp
Addition of infinite branching datatypes
1994-07-27, by lcp
added experimental add_defns (actually should be moved somewhere else);
1994-07-27, by wenzelm
Misc minor updates
1994-07-26, by lcp
Axiom of choice, cardinality results, etc.
1994-07-26, by lcp
Axiom of choice, cardinality results, etc.
1994-07-26, by lcp
added IMP
1994-07-21, by nipkow
Initial revision
1994-07-21, by nipkow
Initial revision
1994-07-21, by nipkow
fixed comment: "(| _ : _ |)" to "OFCLASS(_, _)"
1994-07-20, by wenzelm
*** empty log message ***
1994-07-18, by nipkow
added init_thy_reader and removed extend_theory
1994-07-18, by nipkow
added thy_name to Datatype_Fun's parameter
1994-07-15, by clasohm
added check for concistency of filename and theory name;
1994-07-15, by clasohm
added function mapst
1994-07-15, by clasohm
added functor signature constraint;
1994-07-14, by wenzelm
minor internal renamings;
1994-07-14, by wenzelm
changed syntax "(| _ : _ |)" to "OFCLASS(_, _)";
1994-07-14, by wenzelm
indentation and renaming of rules
1994-07-13, by lcp
minor updates
1994-07-12, by lcp
chain_tac: deleted; just use etac mp
1994-07-12, by lcp
Improved error checking
1994-07-12, by lcp
new cardinal arithmetic developments
1994-07-12, by lcp
removed flatten_typ and replaced add_consts by add_consts_i
1994-07-12, by clasohm
Corrected HOL.tex
1994-07-12, by nipkow
added datatype section
1994-07-12, by nipkow
included rail.sty
1994-07-12, by nipkow
Initial revision
1994-07-11, by nipkow
minor edits
1994-07-11, by lcp
restoring after deletion
1994-07-11, by lcp
minor edits
1994-07-11, by lcp
type constraints
1994-07-11, by nipkow
documented subgoals_tac
1994-07-11, by lcp
New errata list for the documentation
1994-07-11, by lcp
misc updates
1994-07-11, by lcp
removed flatten_term and replaced add_axioms by add_axioms_i
1994-07-11, by clasohm
added () around some of the ::
1994-07-07, by nipkow
changed priority of ::
1994-07-07, by nipkow
exported opt_infix, opt_mixfix parsers;
1994-07-06, by wenzelm
added raw_unify;
1994-07-06, by wenzelm
various minor changes (names and comments);
1994-07-06, by wenzelm
changed comment for const_name
1994-07-06, by clasohm
changed comment only;
1994-07-06, by wenzelm
rewritec now uses trace_thm for it's "rewrite rule from different theory"
1994-07-01, by clasohm
changed syntax of datatype declaration
1994-07-01, by clasohm
replaced extend_theory by new add_* functions;
1994-07-01, by clasohm
added parentheses made necessary by new constrain precedence
1994-06-29, by clasohm
added parentheses made necessary by change of constrain's precedence
1994-06-29, by clasohm
changed precedence of constrain to [4, 0], 3
1994-06-29, by clasohm
FOL/FOL.ML/excluded_middle_tac: new
1994-06-24, by lcp
Pure/tactic/subgoals_tac: new (moved from ZF/Order.ML)
1994-06-24, by lcp
minor tidying up (ordered rewriting in Integ.ML)
1994-06-23, by lcp
modifications for cardinal arithmetic
1994-06-23, by lcp
Sara\'s perl script for renaming theory files
1994-06-23, by lcp
Addition of cardinals and order types, various tidying
1994-06-21, by lcp
Various updates and tidying
1994-06-21, by lcp
improved error msg
1994-06-21, by nipkow
Improved error msg "Proved wrong thm"
1994-06-20, by nipkow
parse.ML and scan.ML are now replaced by thy_parse.ML and thy_scan.ML
1994-06-20, by clasohm
Franz Regensburger's changes.
1994-06-20, by nipkow
atomize: borrowed HOL version, which checks for both Trueprop
1994-06-17, by lcp
problem 38 is provable
1994-06-17, by lcp
ordered rewriting applies to conditional rules as well now
1994-06-17, by nipkow
replaced "foldl merge_theories" by "merge_thy_list" in base_on
1994-06-17, by clasohm
added 'subclass' section;
1994-06-16, by wenzelm
base_on: added 'mk_draft' arg;
1994-06-16, by wenzelm
(beta release)
1994-06-16, by wenzelm
added ext_tsig_subclass, ext_tsig_defsort;
1994-06-16, by wenzelm
added add_classrel;
1994-06-16, by wenzelm
replaced extend_theory;
1994-06-09, by wenzelm
added OldMixfix;
1994-06-09, by wenzelm
workaround bug in Type.expand_typ;
1994-06-09, by wenzelm
new datatype 'mixfix' now pervasive (old one still accesible via OldMixfix);
1994-06-09, by wenzelm
restored functor sig;
1994-06-09, by wenzelm
added axclass.ML, Syntax/mixfix.ML, Thy/thy_syn.ML;
1994-06-09, by wenzelm
added signature constraint;
1994-06-01, by wenzelm
removed garbage;
1994-06-01, by wenzelm
restored old functor name;
1994-06-01, by wenzelm
interface for 'user sections';
1994-06-01, by wenzelm
replaced infix also by |>
1994-06-01, by wenzelm
added test for $ISABELLEBIN=source directory, to
1994-06-01, by lcp
Improved error messages
1994-06-01, by lcp
reflected changes in the structure of Thy
1994-06-01, by nipkow
simpset is hidden in a functor now.
1994-05-31, by nipkow
Internale optimization of the simplifier: in case a subterm stays unchanged,
1994-05-29, by nipkow
axiomatic type class 'package' for Pure (alpha version);
1994-05-26, by wenzelm
added "axclass.ML", structure AxClass;
1994-05-26, by wenzelm
added subsort, norm_sort, classes;
1994-05-26, by wenzelm
replaced "logic" by logicC;
1994-05-26, by wenzelm
replaced ext_axtab by new_axioms;
1994-05-26, by wenzelm
added class_triv: theory -> class -> thm (for axclasses);
1994-05-26, by wenzelm
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
1994-05-26, by wenzelm
changed syntax of use_string
1994-05-26, by clasohm
changed use_string's type to string list -> unit because POLY can only
1994-05-26, by clasohm
"Building new grammar" message is no longer displayed by empty_gram
1994-05-26, by clasohm
Modified mk_meta_eq to leave meta-equlities on unchanged.
1994-05-24, by nipkow
thy reader now initialised by init_thy_reader();
1994-05-19, by wenzelm
*** empty log message ***
1994-05-19, by wenzelm
(was Thy/read.ML)
1994-05-19, by wenzelm
*** empty log message ***
1994-05-19, by wenzelm
(replaces Thy/parse.ML and Thy/syntax.ML)
1994-05-19, by wenzelm
(replaces Thy/scan.ML)
1994-05-19, by wenzelm
new datatype theory, supports 'draft theories' and incremental extension:
1994-05-19, by wenzelm
added const_type: sg -> typ option;
1994-05-19, by wenzelm
added print_sign, print_axioms: theory -> unit;
1994-05-19, by wenzelm
support for new style mixfix annotations;
1994-05-19, by wenzelm
added incremental extension functions: extend_log_types, extend_type_gram,
1994-05-19, by wenzelm
added insort_tr, prop_tr' (for axclasses);
1994-05-19, by wenzelm
replaced fix_aprop by prop_tr';
1994-05-19, by wenzelm
added infix op also: 'a * ('a -> 'b) -> 'b;
1994-05-19, by wenzelm
use_thy now uses use_string instead of creating a temporary file
1994-05-19, by clasohm
added use_string: string -> unit to execute ML commands passed in a string
1994-05-19, by clasohm
lookaheads are now computed faster (during the grammar is built)
1994-05-19, by clasohm
extended signature SCANNER by some basic scanners and type lexicon;
1994-05-18, by wenzelm
added logicC: class, logicS: sort;
1994-05-18, by wenzelm
added make, dest, extend_new;
1994-05-18, by wenzelm
fixed a bug in syntax_error, added "Building new grammar" message;
1994-05-17, by clasohm
syntax_error now checks precedences when computing expected tokens
1994-05-13, by clasohm
FOL/simpdata: added etac FalseE in setsolver call. Toby: "now that the
1994-05-13, by lcp
make-all-poly, make-all-nj: restored to main directory as examples
1994-05-13, by lcp
changed implode to ^
1994-05-11, by clasohm
moved 'filter is_xid' in syn_ext
1994-05-11, by clasohm
syntax_error now removes duplicate tokens in its output and doesn't
1994-05-09, by clasohm
ZF/indrule/mk_pred_typ: corrected pattern to include Abs, allowing it to
1994-05-06, by lcp
renaming/removal of filenames to correct case
1994-05-06, by lcp
renaming/removal of filenames to correct case
1994-05-06, by lcp
renaming/removal of filenames to correct case
1994-05-06, by lcp
improved syntax error:
1994-05-06, by clasohm
CTT.ML/SumE_fst,SumE_snd: tidied
1994-05-04, by lcp
Bool.ML: replaced many rewrite_goals_tac calls by prove_goalw
1994-05-04, by lcp
final Springer version
1994-05-03, by lcp
post-CRC corrections
1994-05-03, by lcp
post-CRC corrections
1994-05-03, by lcp
post-CRC corrections
1994-05-03, by lcp
post-CRC corrections
1994-05-03, by lcp
CTT/Arith.ML: replaced many rewrite_goals_tac calls by prove_goalw
1994-05-03, by lcp
removal of obsolete type-declaration syntax
1994-05-03, by lcp
removal of obsolete type-declaration syntax
1994-05-03, by lcp
removal of obsolete type-declaration syntax
1994-05-03, by lcp
post-CRC corrections
1994-05-03, by lcp
post-CRC corrections
1994-05-03, by lcp
post-CRC corrections
1994-05-03, by lcp
changed translation of type applications according to new grammar;
1994-05-02, by wenzelm
added many more filenames to FILES and EX_FILES
1994-04-27, by lcp
made a few cosmetic changes
1994-04-26, by clasohm
final Springer copy
1994-04-25, by lcp
final Springer copy
1994-04-25, by lcp
renamed theory files
1994-04-24, by clasohm
fixed a small bug
1994-04-24, by clasohm
changed convention for theory file names: they now have to consist of the
1994-04-24, by clasohm
renamed theory files
1994-04-22, by clasohm
renamed theory files
1994-04-22, by clasohm
renamed theory files
1994-04-22, by clasohm
renamed theory files
1994-04-22, by clasohm
renamed theory files
1994-04-22, by clasohm
renamed theory files
1994-04-22, by clasohm
final Springer copy
1994-04-22, by lcp
final Springer copy
1994-04-22, by lcp
final Springer copy
1994-04-22, by lcp
changed the way a grammar is generated to allow the new parser to work;
1994-04-22, by clasohm
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
penultimate Springer draft
1994-04-15, by lcp
restored the signature constraint :THM
1994-04-06, by lcp
modifications towards final draft
1994-04-04, by lcp
modifications towards final draft
1994-04-04, by lcp
changed lists and added "let" and "case"
1994-03-30, by nipkow
Changed term ordering for permutative rewrites to be AC-compatible.
1994-03-27, by nipkow
revisions to first Springer draft
1994-03-24, by lcp
added section on type synonyms
1994-03-24, by nipkow
minor problems
1994-03-24, by nipkow
added \iflabelundefined
1994-03-24, by lcp
removed inconsistency with new HOL version
1994-03-24, by nipkow
Franz fragen
1994-03-24, by nipkow
structural induction for strict lists
1994-03-24, by nipkow
Franz fragen
1994-03-24, by nipkow
revisions to first Springer draft
1994-03-24, by lcp
have broken line
1994-03-23, by nipkow
final CADE version
1994-03-23, by lcp
first draft of Springer volume
1994-03-23, by lcp
first draft of Springer volume
1994-03-23, by lcp
first draft of Springer volume
1994-03-23, by lcp
changed "." to "$" and added parentheses to eliminate ambiguity
1994-03-22, by clasohm
changed "." to "$" to eliminate ambiguity
1994-03-22, by clasohm
Implemented "ordered rewriting": rules which merely permute variables, such
1994-03-22, by nipkow
first draft of Springer book
1994-03-21, by lcp
first draft of Springer book
1994-03-21, by lcp
first draft of Springer book
1994-03-21, by lcp
First draft of Springer book
1994-03-19, by lcp
new type declaration syntax instead of numbers
1994-03-17, by lcp
FOL/simpdata: tidied
1994-03-17, by lcp
CTT/ex/elim.ML: in the two proofs of Axiom of Choice, changed X-->Y to PROD
1994-03-17, by lcp
CCL/ccl.ML/po_refl_iff_T: deleted reference to make_iff_T
1994-03-17, by lcp
Improved layout for inductive defs
1994-03-17, by lcp
adapted type definition to new syntax
1994-03-17, by clasohm
fixed misfeature in Sign.extend: types of consts were read wrt. the new syntax;
1994-03-04, by wenzelm
changed "x" to "uu" for implicit name of the
1994-03-03, by lcp
update towards LNCS
1994-03-01, by nipkow
deleted a comment
1994-03-01, by nipkow
*** empty log message ***
1994-02-26, by nipkow
improved explode_tr;
1994-02-21, by wenzelm
minor update because HOL-lemma changed
1994-02-16, by nipkow
tactic/make_elim_preserve: recoded to avoid using lift_inst_rule. Instead
1994-02-16, by lcp
moved 'unlink ".tmp.ML"' away from 'use ".tmp.ML"' to try to fix a bug with SML
1994-02-16, by clasohm
double_complement_Un: new
1994-02-14, by lcp
*** empty log message ***
1994-02-09, by wenzelm
improved eq_sg;
1994-02-08, by wenzelm
added eq_set;
1994-02-08, by wenzelm
correction to cut tactics
1994-02-04, by lcp
no longer removes *.z
1994-02-03, by lcp
now makes HOLCF
1994-02-03, by lcp
added strs, big_list, writeln;
1994-02-03, by wenzelm
added simple_string_of_typ, simple_pprint_typ;
1994-02-03, by wenzelm
added type 'syntax';
1994-02-03, by wenzelm
minor internal changes;
1994-02-03, by wenzelm
syntax for type abbreviations;
1994-02-03, by wenzelm
(this is a preliminary release)
1994-02-03, by wenzelm
added if_none, parents, commas, gen_duplicates, duplicates, assoc2;
1994-02-03, by wenzelm
replaced pprint_sg by Sign.pprint_sg;
1994-02-03, by wenzelm
replaced eq_sg by Sign.eq_sg;
1994-02-03, by wenzelm
removed eq_sg, pprint_sg, print_sg (now in sign.ML);
1994-02-03, by wenzelm
major cleanup;
1994-02-03, by wenzelm
extend_theory: changed type of "abbrs" arg;
1994-02-03, by wenzelm
made error message "file not found" more informative
1994-02-02, by clasohm
case was renamed to sum_case
1994-01-26, by nipkow
added is_empty: env -> bool, minidx: env -> int option;
1994-01-24, by wenzelm
added HOLCF
1994-01-20, by nipkow
removed square and fact
1994-01-20, by nipkow
HOLCF examples
1994-01-19, by nipkow
Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
1994-01-19, by nipkow
commented out sig constraint of functor (for debugging purposes);
1994-01-19, by wenzelm
changed SYNTAX_FILES;
1994-01-19, by wenzelm
contains remaining parts of xgram.ML and extension.ML;
1994-01-19, by wenzelm
minor internal changes;
1994-01-19, by wenzelm
MAJOR INTERNAL CHANGE: extend and merge operations of syntax tables
1994-01-19, by wenzelm
MAJOR INTERNAL CHANGE: extend and merge operations of syntax tables
1994-01-19, by wenzelm
added some utils: commas, breaks, fbreaks, block, parents, list, str_list;
1994-01-19, by wenzelm
cosmetic changes;
1994-01-19, by wenzelm
minor cleanup;
1994-01-19, by wenzelm
major cleanup and reorganisation;
1994-01-19, by wenzelm
corrected comment
1994-01-18, by lcp
Updated refs to old Sign functions
1994-01-18, by lcp
Many other files modified as follows:
1994-01-18, by lcp
Pure: MAJOR CHANGE. Moved ML types ctyp and cterm and their associated
1994-01-18, by lcp
some optimizations of Larry's
1994-01-18, by nipkow
corrected comments
1994-01-14, by lcp
corrected comments
1994-01-14, by lcp
optimized net for matching of abstractions to speed up simplifier
1994-01-14, by nipkow
moved misplaced comment
1994-01-11, by nipkow
removed Syntax/parse_tree.ML;
1994-01-11, by wenzelm
optimized the number of eta-contractions in rewriting
1994-01-11, by nipkow
added a check for existence of a temporary file before removing it
1994-01-10, by clasohm
used unlink for delete_files instead of calling rm
1994-01-10, by clasohm
commented out sig constraint of functor (for debugging purposes);
1994-01-10, by wenzelm
ZF/perm/image_comp: new
1994-01-07, by lcp
got rid of METAHYPS due to the change of the basic simplification routines
1994-01-05, by nipkow
adapted a proof to the new solver (see change of FOL/simpdata.ML)
1994-01-05, by nipkow
updated solver of FOL_ss. see change of HOL/simpdata.ML
1994-01-05, by nipkow
added new parameter to the simplification tactics which indicates if
1994-01-05, by nipkow
added lexical class of type variables
1994-01-05, by nipkow
shortened msg
1994-01-05, by nipkow
added fake_cterm_of to speed up rewriting
1994-01-04, by nipkow
commented out sig constraint of functor (for debugging purposes);
1994-01-04, by wenzelm
changed tracing of simplifier
1994-01-04, by nipkow
optimized simplifier - signature of rewritten term stays constant
1994-01-02, by nipkow
added "Reading thy-File" message
1993-12-30, by clasohm
added subsig: sg * sg -> bool to test if one signature is contained in another.
1993-12-30, by nipkow
added sys_error;
1993-12-29, by wenzelm
fixed a bug in update/next_level which occured when a child wasn't loaded
1993-12-22, by clasohm
added empty type-abbr field to extend_theory
1993-12-21, by nipkow
added []-field to extend_theory: no type abbreviations.
1993-12-21, by nipkow
Added []-field to extend_theory to accomodate type abbreviations.
1993-12-21, by nipkow
Necessary changes to accomodate type abbreviations.
1993-12-21, by nipkow
pretty_thm is now exported;
1993-12-21, by wenzelm
new section for equality properties
1993-12-21, by lcp
Updated read_insts to approximate simultaneous type checking of substitution
1993-12-14, by nipkow
added isabelle-users paragraph
1993-12-13, by lcp
added mention of simplifier, splitter, hypsubst
1993-12-13, by lcp
new year
1993-12-13, by lcp
updated instantiate to deal with type clashes
1993-12-10, by nipkow
ZF/equalities/SUM_eq_UN: new
1993-12-10, by lcp
Pure/tactic/compose_inst_tac: when catching exception THM, prints the
1993-12-10, by lcp
deleted harmful basify, which pulled rewrite rules down to base type.
1993-12-09, by nipkow
added rep_tsig
Isabelle93
1993-12-06, by nipkow
last minute changes, eg literal tokens -> delimiters and valued tokens ->
1993-12-06, by nipkow
ZF/univ/in_Vfrom_limit: new
1993-12-06, by lcp
ZF/ord/Ord_Un,Ord_Int,Un_upper1_le,Un_upper2_le: new
1993-12-06, by lcp
Typos and style
1993-12-06, by nipkow
Changed Acknowledgements
1993-12-03, by lcp
Acknowledged Carsten Clasohm
1993-12-03, by lcp
New distributive laws for Sigma and UN
1993-12-03, by lcp
removal of amssymbols.sty and lcp.sty; addition of iman.sty
1993-12-02, by lcp
ZF/ex/ROOT: changed many time_use calls to time_use_thy or else deleted
1993-12-01, by lcp
minor corrections
1993-12-01, by lcp
new references
1993-12-01, by lcp
now inspects FOLP_build_completed
1993-12-01, by lcp
now declares FOLP_build_completed
1993-12-01, by lcp
*** empty log message ***
1993-11-30, by wenzelm
*** empty log message ***
1993-11-30, by wenzelm
ZF/ex/llist_eq/lleq_Int_Vset_subset_lemma,
1993-11-30, by lcp
changed split_filename, remove_ext;
1993-11-30, by wenzelm
*** empty log message ***
1993-11-30, by wenzelm
ZF/quniv/QPair_Int_Vset_subset_UN: new, isolates key argument of many
1993-11-30, by lcp
extend: cleaned up, adapted for new Syntax.extend;
1993-11-29, by wenzelm
*** empty log message ***
1993-11-29, by wenzelm
added (partial) extend_tables;
1993-11-29, by wenzelm
changed datatype ext;
1993-11-29, by wenzelm
improved comments;
1993-11-29, by wenzelm
added SCANNER;
1993-11-29, by wenzelm
added Scanner;
1993-11-29, by wenzelm
added logical_types
1993-11-29, by nipkow
improved comments;
1993-11-29, by wenzelm
added equal, not_equal: ''a -> ''a -> bool
1993-11-29, by wenzelm
Minor edits to discussion of use_thy
1993-11-26, by lcp
Correction to eta-contraction; thanks to Markus W.
1993-11-26, by lcp
Correction to page 16; thanks to Markus W.
1993-11-26, by lcp
Corrected errors found by Marcus Wenzel.
1993-11-26, by lcp
changed some names and deleted *NORMALIZED*
1993-11-25, by nipkow
corrected obvious errors;
1993-11-25, by wenzelm
corrected obvious errors;
1993-11-25, by wenzelm
*** empty log message ***
1993-11-25, by wenzelm
corrected some obvious errors;
1993-11-25, by wenzelm
changed beginning of "Reading a new theory", added index "automatic loading"
1993-11-25, by clasohm
corrected trivial typo;
1993-11-25, by wenzelm
corrected trivial typo;
1993-11-25, by wenzelm
fixed a bug in get_filenames, changed output of use_thy
1993-11-25, by clasohm
asm_full_simp_tac now fails if there are no subgoals
1993-11-25, by nipkow
added subsection 'Classes and types';
1993-11-25, by wenzelm
added Syntax.read_typ;
1993-11-25, by wenzelm
Sign.extend: Syntax.extend now called with read_ty;
1993-11-25, by wenzelm
removed section 'Classes and types';
1993-11-25, by wenzelm
added index commands, removed last paragraph of "Using Poly/ML"
1993-11-25, by clasohm
changed itmath trickery to be compatible with NFSS (itmath.sty)
1993-11-23, by nipkow
minor changes
1993-11-22, by nipkow
added chapter "Defining Theories" and made changes for new Readthy functions
1993-11-22, by clasohm
*** empty log message ***
1993-11-22, by wenzelm
*** empty log message ***
1993-11-22, by wenzelm
various minor changes;
1993-11-22, by wenzelm
Fixed bug in rewriter (fun impc) discovered by Marcus Moore.
1993-11-22, by nipkow
Reformatting of SIMPLIFIER figure
1993-11-19, by lcp
less
more
|
(0)
-480
+480
+1000
+3000
+10000
+30000
tip