Mercurial
Mercurial
>
repos
>
Old_HOL
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-120
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.
minor cleanup, added 'axclass', 'instance', 'syntax', 'defs' sections;
1994-09-21, by wenzelm
Definition of C was not truly prim rec because C was called inside Gamma
1994-09-16, by nipkow
improved error reporting for primrec
1994-09-15, by nipkow
replaced lookup_const by Sign.const_type;
Isabelle94
1994-09-14, by wenzelm
Allowed string as function name in primrec header
1994-09-11, by nipkow
{HOL,ZF}/indrule/quant_induct: replaced ssubst in eresolve_tac by
1994-09-08, by lcp
HOL/IMP/Equiv/bexp_iff: split proof into separate directions, to be faster
1994-09-07, by lcp
changed names
1994-09-06, by nipkow
Converted rules to primrecs
1994-09-06, by nipkow
corrected comment re treatment of types such as (bool*bool)*bool
1994-09-06, by lcp
HOL/ex/PropLog.thy: tidied
1994-09-06, by lcp
HOL/ind_syntax/factors: now returns only factors in the product type that
1994-09-06, by lcp
Added IMP, which necessiated changes in intr_elim.tex (mk_cases).
1994-08-31, by nipkow
Renamed a few types and vars
1994-08-31, by nipkow
Equivalence of op. and den. sem. for simple while language.
1994-08-31, by nipkow
Updated PL to PropLog using Larrys ind. defs.
1994-08-30, by nipkow
New version of datatype.ML with primrec (Norbert).
1994-08-30, by nipkow
INSTALLATION OF INDUCTIVE DEFINITIONS
1994-08-25, by lcp
INSTALLATION OF INDUCTIVE DEFINITIONS
1994-08-25, by lcp
Subst/UTerm: updated for inductive defs; streamlined proofs
1994-08-24, by lcp
HOL/ex/MT.thy: now mentions dependence upon Sum.thy
1994-08-22, by lcp
new header & minor changes
1994-08-22, by lcp
changed defn to def
1994-08-22, by lcp
HOL/Sum.thy: generalized the type of Part
1994-08-22, by lcp
replaced add_defns_i by add_defs_i;
1994-08-19, by wenzelm
HOL/Trancl.thy: depends upon Prod
1994-08-19, by lcp
HOL/Makefile, ROOT: updated for new .thy files
1994-08-19, by lcp
HOL/Ord.thy,.ML: files now have header comments
1994-08-19, by lcp
HOL/Sum: added disjoint sum of two sets as the plus operator, since + is
1994-08-19, by lcp
HOL/subset.thy, equalities.thy, mono.thy: new
1994-08-19, by lcp
HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
1994-08-19, by lcp
HOL/ex/Term, Simult: updated for new Split
1994-08-18, by lcp
HOL/List: rotated arguments of List_case, list_case
1994-08-18, by lcp
HOL/Prod: swapped args of split and simplified
1994-08-18, by lcp
HOL/Univ: swapped args of split and simplified
1994-08-18, by lcp
HOL/Sexp: rotated arguments of Sexp_case
1994-08-18, by lcp
HOL/Nat: rotated arguments of nat_case; added translation for case macro
1994-08-18, by lcp
HOL/Trancl: comp_cs is based upon prod_cs; tidied proofs
1994-08-18, by lcp
HOL/Sum: rotated arguments of sum_case; added translation for case macro
1994-08-18, by lcp
HOL/Subst/AList: swapped args of split and simplified
1994-08-18, by lcp
HOL/LList: swapped args of split and simplified
1994-08-18, by lcp
allow long_id for reference to type in primrec.
1994-08-16, by nipkow
Cleaned up code.
1994-08-15, by nipkow
Used the new primitive recursive functions format for thy-files
1994-08-13, by nipkow
Added primitive recursive functions (Norbert Voelker's code) to the datatype
1994-08-13, by nipkow
renamed meta_obj_reflection meta_eq_to_obj_eq.
1994-08-03, by nipkow
exposed meta_obj_reflection
1994-08-02, by nipkow
added a new example due to Robin Arthan
1994-07-27, by lcp
HOL/Makefile: now test depends upon SUBST_FILES
1994-07-21, by lcp
Lots of simplifications
1994-07-15, by nipkow
added val eq_sym_conv = prover "(x=y) = (y=x)";
1994-07-15, by nipkow
fixed indentation
1994-07-12, by lcp
Integrated PL0.thy into PL.thy
1994-07-08, by nipkow
Hidden dtK and Impossible with a "local" clause
1994-07-08, by nipkow
added mixfix annotations to constructor declarations
1994-07-08, by clasohm
added parentheses made necessary by change of constrain's precedence
1994-06-29, by clasohm
HOL/Nat/less_asym: renamed from less_anti_sym
1994-06-24, by lcp
HOL/WF/wf_asym: renamed from wf_anti_sym
1994-06-24, by lcp
added prefix to name of induct axiom
1994-06-20, by clasohm
Datatype -> Datatype.ML
1994-06-20, by nipkow
HOL/Arith/add_left_commute: tidied
1994-06-17, by lcp
HOL/HOL.ML/notE: tidied the proof
1994-06-17, by lcp
HOL/List/map_append,map_compose: new
1994-06-17, by lcp
HOL/ex/NatSum: added another example
1994-06-17, by lcp
adopted to new datatype definition method
1994-06-17, by clasohm
datatypes must now be defined using a thy file section
1994-06-17, by clasohm
Added set comprehension as a syntactic abbreviation:
1994-06-15, by nipkow
added test for $ISABELLEBIN=source directory, to
1994-06-01, by lcp
HOL/Arith: definition of diff now uses pred, not nat_rec
1994-05-25, by lcp
HOL/equalities: added some identities from ZF/equalities
1994-05-25, by lcp
HOL/HOL.ML/notE: tidied
1994-05-25, by lcp
thy reader now initialised by init_thy_reader();
1994-05-19, by wenzelm
HOL/Prod/pair_eq: renamed to Pair_fst_snd_eq
1994-05-13, by lcp
removal of obsolete type-declaration syntax
1994-05-03, by lcp
removal of obsolete type-declaration syntax
1994-05-03, by lcp
renamed theory files
isa94
1994-04-24, by clasohm
renamed theory files
1994-04-22, by clasohm
tidied definitions and proofs
1994-04-21, by lcp
HOL/arith.ML/plus_leD1: tidied
1994-04-21, by lcp
changed defns in hol.thy from = to ==
1994-04-19, by nipkow
Now simplifies before the induction
1994-04-06, by lcp
@ now associates to the right, just like #, in order to avoid loss of
1994-03-30, by nipkow
Added some sums.
1994-03-27, by nipkow
integrated permutative rewriting
1994-03-27, by nipkow
used new field "simps" of Datatype
1994-03-22, by nipkow
new field "simps" added
1994-03-22, by nipkow
added dependency on datatype.ML
1994-03-22, by nipkow
Updated simpsets and a few proofs.
1994-03-22, by nipkow
Updated simpsets and a few proofs.
1994-03-22, by nipkow
Used Datatype functor to define propositional logic terms.
1994-03-22, by nipkow
simplified some proofs using ordered rewriting.
1994-03-22, by nipkow
used ordered rewriting to simplify some proofs
1994-03-22, by nipkow
ML-like datatype decalaration facility. Axiomatic.
1994-03-18, by nipkow
added use_thy"Datatype"
1994-03-18, by nipkow
new type declaration syntax instead of numbers
1994-03-17, by lcp
HOL/equalities/Int_Union_image, Un_Inter_image: renamed Int_Union, Un_Inter
1994-03-17, by lcp
adapted type definition to new syntax
1994-03-17, by clasohm
changed "." to "$" and Cons to infix "#" to eliminate ambiguity
1994-03-02, by clasohm
typo in comment
1994-02-24, by nipkow
some more sorting algorithms
1994-02-23, by nipkow
added more lemmas (also to nat_ss)
1994-02-16, by nipkow
deleted duplicate rewrite rules
1994-02-15, by nipkow
added etac FalseE to the simplifier's solver.
1994-02-15, by nipkow
added translations for "case xs of"
1994-02-12, by nipkow
added ::bool in the defn of True.
1994-02-11, by nipkow
Introduction of various new lemmas and of case_tac.
1994-02-03, by nipkow
id -> idt in type of @filter and @Alls
1994-01-27, by nipkow
sum: renamed case to sum_case
1994-01-26, by nipkow
changed header
1994-01-24, by nipkow
Verification of quicksort
1994-01-24, by nipkow
added qsort
1994-01-24, by nipkow
added conj_assoc to HOL_ss
1994-01-24, by nipkow
commented imageE
1994-01-14, by lcp
added let_weak_cong
1994-01-07, by nipkow
added pair_eq
1994-01-07, by nipkow
modified solver of HOL_ss to take the new simplifier into account: the thm to
1994-01-05, by nipkow
added new rewrite rules to arith_ss
1994-01-05, by nipkow
shortened use_thy section taking advantage of dependencies
1994-01-04, by nipkow
added x ~: {} and x : insert(y,A) = ...
1993-12-30, by nipkow
added Pair_eq to pair_ss in prod.ML
1993-12-22, by nipkow
less
more
|
(0)
-120
tip