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.
Enforced partial evaluation of mk_case_split_tac.
1995-03-08, by nipkow
Enforced partial evaluation of mk_case_split_tac
1995-03-08, by nipkow
Added dependencies on files in Provers
1995-03-08, by nipkow
Added pretty-printing coments
1995-03-08, by nipkow
*** empty log message ***
1995-03-07, by nipkow
*** empty log message ***
1995-03-07, by nipkow
Hoare logic
1995-03-07, by nipkow
Changed Univ to Datatype in parents
1995-03-07, by lcp
Replaced rules by defs. Also got rid of tyconstU by
1995-03-07, by lcp
Replaced rules by defs
1995-03-07, by lcp
Got rid of exvarU and constU by
1995-03-07, by lcp
Deleted constQU, exvarQU, expQU by including Const,
1995-03-07, by lcp
Replaced rules by defs
1995-03-07, by lcp
Moved declarations of @QSUM and <*> to a syntax section.
1995-03-07, by lcp
Moved declaration of ~= to a syntax section
1995-03-07, by lcp
replaced Pure by ProtoPure
1995-03-03, by clasohm
fixed a bug in infer_types/exn_type_msg
1995-03-03, by clasohm
new version of HOL/Integ with curried function application
1995-03-03, by clasohm
new version of HOL/IMP with curried function application
1995-03-03, by clasohm
new version of HOL with curried function application
1995-03-03, by clasohm
added CPure (curried functions) and ProtoPure (ancestor of Pure and CPure)
1995-03-03, by clasohm
added declaration of syntactic const "_abs";
1995-03-02, by wenzelm
Added initial /bin/csh line and comments
1995-02-28, by lcp
No longer calls maketest; instead, the Makefile writes the file
1995-02-28, by lcp
Uses "suffix substitution" to shorten macro definitions.
1995-02-28, by lcp
Re-organised to perform the tests independently. Now test
1995-02-28, by lcp
New example by Jacob Frost, tidied by lcp
1995-02-28, by lcp
New example by Jacob Frost, tidied by lcp
1995-02-27, by lcp
Now prove_goalw_cterm calls print_sign_exn_unit, so that the rest
1995-02-27, by lcp
Updated the "version" variable (which was never done for
1995-02-27, by lcp
Redefined functions to suppress redundant leading 0s and 1s
1995-02-27, by lcp
new in mixfix annotations: "' " (quote space) separates delimiters without
1995-02-27, by wenzelm
Added the exception handler
1995-02-27, by lcp
intro_tacsf now includes subsetI as an introduction rule. It is
1995-02-27, by lcp
Updated comment about list_subset_univ and list_into_univ.
1995-02-27, by lcp
exit: new, for use in Makefiles
1995-02-27, by lcp
Redefined arithmetic to suppress redundant leading 0s and 1s
1995-02-27, by lcp
Added integer numerals (mostly due to Markus Wenzel)
1995-02-27, by lcp
Proved zadd_left_commute and zmult_left_commute to define
1995-02-27, by lcp
New shell script for finding orphan .ML files (those with no
1995-02-27, by lcp
added ExcludeThm; cleaned up Makefile; fixed isalpha bug (replaced by isalnum)
1995-02-24, by clasohm
added check "length ts > 1" before printing ambiguity warning in infer_types
1995-02-17, by clasohm
Improved test for looping rewrite rules.
1995-02-16, by nipkow
replaced pair_ss by prod_ss
1995-02-15, by regensbu
Improved check for looping conditional rewrite rules.
1995-02-08, by nipkow
ID for the file
1995-02-07, by regensbu
ID for the file
1995-02-07, by regensbu
'get ID update working'
1995-02-07, by regensbu
CVS:
1995-02-07, by regensbu
CVS:
1995-02-07, by regensbu
added qed, qed_goal[w]
1995-02-07, by clasohm
added specification of csh as script interpreter
1995-02-03, by clasohm
simplified elimination of chain productions
1995-02-02, by clasohm
binder: optional body pri now [bracketted];
1995-01-27, by wenzelm
improved read_xrules: patterns no longer read twice;
1995-01-27, by wenzelm
*** empty log message ***
1995-01-27, by wenzelm
instance: now automatically includes defs of current thy node as witnesses;
1995-01-27, by wenzelm
binder: optional body pri now [bracketted];
1995-01-27, by wenzelm
added documentation of pwd
1995-01-27, by clasohm
renamed Sign.ambiguity_level to Syntax.ambiguity_level
1995-01-27, by clasohm
moved ambiguity_level from sign.ML to Syntax/syntax.ML
1995-01-27, by clasohm
moved ambiguity_level to Syntax/syntax.ML
1995-01-27, by clasohm
added documentation of Sign.ambiguity_level
1995-01-26, by clasohm
added reference variable ambiguity_level to control ambiguity warnings
1995-01-26, by clasohm
changed due to new .bib files
1995-01-25, by lcp
added optional body priority to binder declaration
1995-01-24, by clasohm
Under RS added cross reference to bind_thm
1995-01-24, by lcp
documented slow_tac, slow_best_tac, depth_tac, deepen_tac
1995-01-24, by lcp
removed mention of FOL_dup_cs
1995-01-24, by lcp
\bibliography now includes crossref.bib
1995-01-24, by lcp
updates for Isabelle94-2
1995-01-24, by lcp
simplified get_thm a bit
1995-01-23, by clasohm
Replaced ordermap_z_lepoll by ordermap_z_lt, which is
1995-01-20, by lcp
README: Now documents to Tools directory
1995-01-20, by lcp
Deleted semicolon at the end of the qed_goal line, which was preventing
1995-01-20, by lcp
some cosmetic changes
1995-01-19, by nipkow
added documentation of bind_thm, qed, qed_goal, get_thm, thms_of
1995-01-19, by clasohm
added optional precedence for body of binder;
1995-01-18, by clasohm
quite a lot of minor and major revisions (inspecting theories, read_axm,
1995-01-18, by wenzelm
empty_def typo
Isabelle94-2
1995-01-13, by lcp
Proved comp_lam.
1995-01-13, by lcp
Corrected indexing of *datatype
1995-01-13, by lcp
prove_fun now includes equalityI. Added the rewrite rules
1995-01-12, by lcp
Proved sum_bij, sum_ord_iso_cong, prod_bij,
1995-01-12, by lcp
Proved case_cong and case_case.
1995-01-12, by lcp
Renamed single_fun to singleton_fun.
1995-01-12, by lcp
Now also depends upon equalities.thy, allowing use of the
1995-01-12, by lcp
Added singleton_iff, Sigma_empty1, Sigma_empty2, Collect_simps
1995-01-12, by lcp
Removed spurious comment about eq_cs
1995-01-12, by lcp
Moved theorems Ord_cases_lemma and Ord_cases to Ordinal.ML
1995-01-12, by lcp
Now depends upon Bool, so that 1 and 2 are defined
1995-01-12, by lcp
Moved theorems Ord_cases_lemma and Ord_cases here from Univ,
1995-01-12, by lcp
Added constants Ord_alt, ++, **
1995-01-12, by lcp
Proved equivalence of Ord and Ord_alt. Proved
1995-01-12, by lcp
Proved ord_isoI, ord_iso_refl. Simplified proof of
1995-01-11, by lcp
Proved cadd_cmult_distrib.
1995-01-11, by lcp
Now proof of Ord_jump_cardinal uses
1995-01-11, by lcp
Added Krzysztof's theorem LeastI2. Proof of sum_eqpoll_cong
1995-01-11, by lcp
pretty_gram: now sorts productions;
1995-01-11, by wenzelm
removed print_sign, print_axioms;
1995-01-11, by wenzelm
slightly changed OFCLASS syntax;
1995-01-11, by wenzelm
fixed minor typos;
1995-01-02, by wenzelm
added;
1995-01-02, by wenzelm
RepFun_eq_0_iff, RepFun_0: new
1994-12-23, by lcp
Moved Transset_includes_summands and Transset_sum_Int_subset
1994-12-23, by lcp
Re-indented declarations; declared the number 2
1994-12-23, by lcp
Added Krzysztof's theorems irrefl_converse, trans_on_converse,
1994-12-23, by lcp
Added Krzysztof's theorems irrefl_rvimage, trans_on_rvimage,
1994-12-23, by lcp
singleton_iff: new
1994-12-23, by lcp
Proved cons_lepoll_consD, succ_lepoll_succD, cons_eqpoll_consD,
1994-12-23, by lcp
Added Krzysztof's constants lesspoll and Finite
1994-12-23, by lcp
Added Krzysztof's theorem pred_Memrel
1994-12-23, by lcp
Moved Transset_includes_summands and Transset_sum_Int_subset to
1994-12-23, by lcp
natE0: deleted, since unused
1994-12-23, by lcp
Changed succ(1) to 2 in in_VLimit, two_in_univ
1994-12-23, by lcp
csquare_rel_def: renamed k to K
1994-12-23, by lcp
inj_apply_equality: new
1994-12-23, by lcp
Added Krzysztof's theorems subst_elem, not_emptyI, not_emptyE
1994-12-23, by lcp
empty_fun: generalized from -> to Pi
1994-12-23, by lcp
Changed succ(1) to 2 in cmult_2; Simplified proof of InfCard_is_Limit
1994-12-23, by lcp
Added Krzysztof's theorems singleton_eq_iff, fst_type, snd_type
1994-12-23, by lcp
Added Krzysztof's theorem disj_imp_disj
1994-12-23, by lcp
Id: marker.
1994-12-21, by lcp
Added comments and Id: marker.
1994-12-21, by lcp
Added comments and Id: marker.
1994-12-21, by lcp
Tools description, largely taken from ../README
1994-12-21, by lcp
Moved description of tools to Tools/README
1994-12-21, by lcp
ord_iso_rvimage: new
1994-12-20, by lcp
Moved well_ord_Memrel, lt_eq_pred, Ord_iso_implies_eq_lemma,
1994-12-20, by lcp
qed is a utility that makes ML files store the defined theories in Isabelle's
1994-12-20, by clasohm
Simplified proof of ord_iso_image_pred using bij_inverse_ss.
1994-12-20, by lcp
Used bind_thm to store domain_rel_subset and range_rel_subset
1994-12-20, by lcp
removed quotes around "Datatype",
1994-12-19, by lcp
removed quotes around "Inductive"
1994-12-19, by lcp
ran expandshort script
1994-12-19, by lcp
ran expandshort script
1994-12-19, by lcp
removed quotes around "Inductive"
1994-12-19, by lcp
added true theory dependencies
1994-12-19, by lcp
ran expandshort script
1994-12-19, by lcp
changed useless "qed" calls for lemmas back to uses of "result",
1994-12-16, by lcp
Defines ZF theory sections (inductive, datatype) at the start/
1994-12-16, by lcp
Added Limit_csucc from CardinalArith
1994-12-16, by lcp
Limit_csucc: moved to InfDatatype and proved explicitly in
1994-12-16, by lcp
put quotation marks around constant "and" because it is a
1994-12-16, by lcp
added thy_syntax.ML
1994-12-16, by lcp
Defines ZF theory sections (inductive, datatype) at the start/
1994-12-16, by lcp
now also depends upon Finite.thy
1994-12-16, by lcp
converse_converse, converse_prod: renamed from
1994-12-16, by lcp
moved congruence rule conj_cong2 to FOL/IFOL.ML
1994-12-16, by lcp
conj_cong2: new congruence rule
1994-12-16, by lcp
case_ss: now built upon ZF/Order/bij_inverse_ss. Deleted
1994-12-15, by lcp
updated comment;
1994-12-15, by lcp
qconverse_qconverse, qconverse_prod: renamed from
1994-12-15, by lcp
well_ord_iso_predE replaces not_well_ord_iso_pred
1994-12-14, by lcp
Ord_iso_implies_eq_lemma: uses well_ord_iso_predE instead of
1994-12-14, by lcp
converse_UN, Diff_eq_0_iff: new
1994-12-14, by lcp
added constants mono_map, ord_iso_map
1994-12-14, by lcp
cardinal_UN_Ord_lt_csucc: added comment
1994-12-14, by lcp
conj_commute,disj_commute: new
1994-12-14, by lcp
changed get_thm to search all parent theories if the theorem is not found
1994-12-14, by clasohm
added bind_thm for theorems defined by "standard ..."
1994-12-14, by clasohm
added any, sprop to pure_types;
1994-12-14, by wenzelm
removed "logic1";
1994-12-14, by wenzelm
removed FOL_Lemmas and IFOL_Lemmas; added qed_goal
1994-12-13, by clasohm
added print_theory that prints stored thms;
1994-12-12, by wenzelm
minor internal changes;
1994-12-09, by wenzelm
improved axioms_of: returns thms as the manual says;
1994-12-09, by wenzelm
removed ZF_Lemmas and added qed_goal
1994-12-09, by clasohm
added warning for already stored theorem to store_thm
1994-12-09, by clasohm
sum_ss: moved down and added the rewrite rules for "case"
1994-12-08, by lcp
leI: added comment
1994-12-08, by lcp
lt_eq_pred, Ord_iso_implies_eq: new, for Kunens Theorem 7.3
1994-12-08, by lcp
sum_ss: deleted because it conflicts with the one in Sum.ML
1994-12-08, by lcp
not_well_ord_iso_pred: removed needless quantifier
1994-12-08, by lcp
UN_upper_cardinal: updated to refer to Card_le_imp_lepoll
1994-12-08, by lcp
sum_lepoll_self, cadd_le_self, prod_lepoll_self,
1994-12-08, by lcp
le_imp_lepoll: renamed to Card_le_imp_lepoll
1994-12-08, by lcp
Card_cardinal_le: new
1994-12-08, by lcp
changed Pure's grammar and the way types are converted to nonterminals
1994-12-08, by clasohm
replaced type_syn by pure_syn in Pure signature
1994-12-08, by clasohm
test_assume_tac: now tries eq_assume_tac on exceptional cases
1994-12-08, by lcp
res_inst_tac: added comments
1994-12-08, by lcp
added qed and qed_goal[w]
1994-12-07, by clasohm
moved first call of store_theory from thy_read.ML to created .thy.ML file
1994-12-07, by clasohm
added bind_thm
1994-12-06, by clasohm
added qed and qed_goal[w]
1994-11-30, by clasohm
added qed_goal for meta_iffD
1994-11-30, by clasohm
replaced "val ... = result()" by "qed ..."
1994-11-30, by clasohm
le_UN_Ord_lt_csucc: added comment
1994-11-29, by lcp
replaced "rules" by "defs"
1994-11-29, by lcp
----------------------------------------------------------------------
1994-11-28, by regensbu
ZF/indrule/mutual_ind_tac: ensured that asm_full_simp_tac ignores any
1994-11-25, by lcp
checks that the recursive sets are Consts before taking
1994-11-25, by lcp
equiv_comp_eq: simplified proof
1994-11-25, by lcp
moved Cantors theorem here from ZF/ex/misc
1994-11-25, by lcp
deepen_tac: modified due to outcome of experiments. Its
1994-11-25, by lcp
added qed_goal[w]
1994-11-25, by clasohm
added blank line
1994-11-25, by lcp
tidied proofs, using fast_tac etc. as much as possible
1994-11-25, by lcp
prove_fun: new; no longer depends upon the version in simpdata.ML
1994-11-25, by lcp
data_domain,Codata_domain: removed replicate; now return one
1994-11-24, by lcp
tidied proofs, using fast_tac etc. as much as possible
1994-11-24, by lcp
added comments on alternative uses of type_intrs/elims
1994-11-24, by lcp
modified for new treatment of mutual recursion
1994-11-24, by lcp
the_equality: more careful use of addSIs and addIs
1994-11-24, by lcp
cons_fun_eq: modified strange uses of classical reasoner
1994-11-24, by lcp
moved Cantors theorem to ZF/ZF.ML and ZF/Perm.ML
1994-11-24, by lcp
moved version of Cantors theorem to ZF/Perm.ML
1994-11-24, by lcp
ZF INDUCTIVE DEFINITIONS: Simplifying the type checking for mutually
1994-11-24, by lcp
ZF/Datatype/datatype_decl: supplies a SINGLE domain for the mutually
1994-11-24, by lcp
updated for new deepen_tac
1994-11-24, by lcp
trivial changes
1994-11-24, by lcp
new reference to HO patterns
1994-11-23, by lcp
Pure/tctical/protect_subgoal: simplified to use Sequence.hd
1994-11-22, by lcp
Pure/term: commented typ_subst_TVars, subst_TVars, subst_Vars, subst_vars
1994-11-22, by lcp
ZF INDUCTIVE DEFINITIONS: Simplifying the type checking for mutually
1994-11-21, by lcp
ZF/intr_elim/elim: now "folds" definitions of the mutually recursive sets!
1994-11-21, by lcp
replaced 'val ... = result();' by 'qed "...";'
1994-11-21, by clasohm
ZF/indrule/mutual_ind_tac: backtracks using DEPTH_SOLVE to be certain of
1994-11-21, by lcp
ZF/EquivClass/congruent_commuteI: uncommented and simplified proof
1994-11-21, by lcp
ZF/ZF.ML/UN_iff, INT_iff: added to the signature
1994-11-21, by lcp
Pure/thm/norm_term_skip: new, for skipping normalization of the context
1994-11-21, by lcp
Pure/sequence: added comment explaining that memoing sequences were found
1994-11-21, by lcp
Pure/envir/norm_term: replaced equality test for [] by null
1994-11-21, by lcp
page 157 erratum
1994-11-21, by lcp
now searches all subdirectories of object-logics
1994-11-21, by lcp
Chnaged simplifier description (lhss)
1994-11-18, by nipkow
added call of store_theory after thy file has been read
1994-11-18, by clasohm
Updated description of valid lhss.
1994-11-18, by nipkow
In ZF, type i has class term, not (just) logic
1994-11-17, by lcp
added check for newlines not enclosed by '\' inside strings
1994-11-14, by clasohm
updated remarks about grammar; added section about ambiguities
1994-11-14, by clasohm
exported 'cat';
1994-11-14, by wenzelm
Pure/tctical/select: now uses cprems_of instead of prems_of and cterm_of:
1994-11-14, by lcp
Pure/drule/cprems_of, cskip_flexpairs, cstrip_imp_prems: new cterm operations
1994-11-14, by lcp
Added month for Coens thesis
1994-11-14, by lcp
removal of FOL_dup_cs
1994-11-11, by lcp
removal of HOL_dup_cs
1994-11-11, by lcp
Provers/hypsubst/REPEATN: deleted; using REPEAT_DETERM_N instead.
1994-11-11, by lcp
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
1994-11-11, by lcp
FOL/intprover/safe_tac: now uses REPEAT_DETERM_FIRST instead of REPEAT_DETERM
1994-11-11, by lcp
argument swaps in HOL
1994-11-11, by lcp
HOL,ZF/Makefile: enclosed multiple "use" calls in parentheses. This
1994-11-10, by lcp
updated pathnames
1994-11-10, by lcp
updated discussion of congruence rules in first section
1994-11-09, by lcp
changed warning for extremely ambiguous expressions
1994-11-09, by clasohm
Pure/goals/prepare_proof/mkresult: now smashes flexflex pairs in the final
1994-11-03, by lcp
ZF/ex/Ramsey,Rmap,misc.ML: modified for new definition of Pi(A,B)
1994-11-03, by lcp
ZF/ex/Ramsey,Rmap,misc.ML: modified for new definition of Pi(A,B)
1994-11-03, by lcp
ZF/Perm/inj_converse_fun: tidied; removed uses of PiI/E
1994-11-03, by lcp
ZF/InfDatatype/fun_Vcsucc: removed use of PiE
1994-11-03, by lcp
ZF/func: tidied many proofs, using new definition of Pi(A,B)
1994-11-03, by lcp
ZF: NEW DEFINITION OF PI(A,B)
1994-11-03, by lcp
ZF/Fixedpt/subset_cs: moved to ZF/subset.ML
1994-11-03, by lcp
ZF/Fixedpt/subset0_cs: moved to ZF/ZF.ML
1994-11-03, by lcp
ZF/domrange/converse_iff: new
1994-11-03, by lcp
ZF/upair/theI2: new
1994-11-03, by lcp
ZF/equalities/domain_converse,range_converse,
1994-11-03, by lcp
ZF/Fixedpt/subset0_cs: moved to ZF/ZF.ML
1994-11-03, by lcp
Cardinal_AC/surj_implies_inj: uses Pi_memberD instead of memberPiE
1994-11-03, by lcp
added warning message
1994-11-03, by clasohm
Provers/classical: now takes theorem "classical" as argument, proves "swap"
1994-11-02, by lcp
Provers/hypsubst: greatly simplified! No longer simulates a
1994-11-02, by lcp
Pure/sign/infer_types/exn_type_msg: new, for more uniform handling of
1994-11-02, by lcp
Modified pattern.ML to perform proper matching of Higher-Order Patterns.
1994-11-02, by nipkow
FOL/FOL/swap: deleted
1994-11-01, by lcp
HOLCF/Ssum3.ML: changed res_inst_tac [("P"... to res_inst_tac [("Pa" in
1994-11-01, by lcp
ZF/ZF.thy: added precedences to @RepFun to disambiguate phrases like {x:A.x:B}
1994-10-31, by lcp
ZF/domrange/image_subset: tidied
1994-10-31, by lcp
ZF/upair/mem_asym,succ_inject: tidied
1994-10-31, by lcp
com1,2: added simplifier calls to remove use of ssubst in fast_tac
1994-10-31, by lcp
Pure/tctical/THEN_ELSE: new
1994-10-31, by lcp
Pure/tactic/build_netpair: now takes two arguments
1994-10-31, by lcp
Pure/sequence/hd,tl: new
1994-10-31, by lcp
Pure/drule/thin_rl: new
1994-10-31, by lcp
FOL/ex/ROOT: now loads mini.ML
1994-10-31, by lcp
FOL/ROOT/FOL_dup_cs: removed as obsolete
1994-10-31, by lcp
FOL/ex/cla: proofs now use deepen_tac instead of best_tac FOL_dup_cs
1994-10-31, by lcp
ZF/ZF/ex1_functional: moved to FOL/ROOT
1994-10-31, by lcp
Miniscope conversoin; example of formula rewriting
1994-10-31, by lcp
ZF/OrderArith/thin: deleted as obsolete
1994-10-31, by lcp
added final newline
1994-10-31, by lcp
added header files; deleted commented-out code
1994-10-31, by lcp
Prepared the code for preservation of bound var names during rewriting. Still
1994-10-28, by nipkow
removed superfluous type_intrs in datatype com.
1994-10-26, by nipkow
simplified syntax of infix continuous functiuons
1994-10-26, by nipkow
strip_quotes now exported;
1994-10-25, by wenzelm
minor change of occs_const in dest_defn;
1994-10-25, by wenzelm
added require_thy;
1994-10-25, by wenzelm
HOL,ZF/IMP/Com.thy: tightening precedences to eliminate syntactic ambiguities.
1994-10-24, by lcp
ZF/intr_elim/elim_rls: now includes Pair_inject, since coinductive
1994-10-21, by lcp
Pure/Unify/IMPROVING "CLEANING" OF FLEX-FLEX PAIRS: Old code would refuse
1994-10-21, by lcp
LK/hardquant/37: deleted call to flexflex_tac: no longer needed
1994-10-21, by lcp
LCF/LCF.thy: the constant VOID had mixfix syntax "()" !! Added quotes.
1994-10-21, by lcp
FOLP/IFOLP.thy: tightening precedences to eliminate syntactic ambiguities.
1994-10-21, by lcp
ZF/Fixedpt/coinduct: modified proof to suppress deep unification
1994-10-19, by lcp
new comments explaining abandoned change
1994-10-19, by lcp
LCF/fix/lfp_is_FIX: modified proof to suppress deep unification
1994-10-19, by lcp
FOL/ex/cla/58: slightly shorter proof
1994-10-19, by lcp
trivial update to reference
1994-10-19, by lcp
CCL/Gfp/coinduct2, coinduct3: modified proofs to suppress deep unification
1994-10-19, by lcp
add_defs: improved error messages;
1994-10-12, by wenzelm
removed old comment;
1994-10-12, by wenzelm
remove _explode, _implode and trfuns;
1994-10-12, by wenzelm
prove_subclass, prove_arity now exported;
1994-10-12, by wenzelm
added is_equals: term -> bool;
1994-10-12, by wenzelm
type_args, opt_witness now exported;
1994-10-12, by wenzelm
AxClass no longer open;
1994-10-12, by wenzelm
{HOL,ZF}/intr_elim/intro_tacsf: now calls DEPTH_SOLVE_1 instead of REPEAT to
1994-10-12, by lcp
{HOL,ZF}/indrule/ind_tac: now calls DEPTH_SOLVE_1 instead of REPEAT, to
1994-10-12, by lcp
fixed infix names in print_translations;
1994-10-12, by wenzelm
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
1994-10-12, by lcp
Minor reference updates
1994-10-12, by lcp
Moving theory LList to ex directory
1994-10-12, by lcp
corrected problems with changed binding power of ::.
1994-10-10, by nipkow
README file
1994-10-10, by nipkow
changed precedences of _constrain (i.e. "::")
1994-10-08, by clasohm
New version
1994-10-06, by nipkow
made major changes to grammar;
Isabelle94-1
1994-10-04, by clasohm
added print_msg;
1994-10-04, by clasohm
Modified termord to take account of the Abs-Abs case.
1994-09-27, by nipkow
improved expand_typ (now handles TVars);
1994-09-26, by wenzelm
exported pretty_sort;
1994-09-26, by wenzelm
added init_pps;
1994-09-26, by wenzelm
added init_database (somewhat experimental);
1994-09-26, by wenzelm
added flag show_no_free_types: bool ref;
1994-09-26, by wenzelm
explode_tr now produces leadings 0s;
1994-09-26, by wenzelm
minor cleanup, added 'syntax' section;
1994-09-21, by wenzelm
now mentions that the sections are available as
1994-09-15, by lcp
removed lookup_const (use Sign.const_type instead);
Isabelle94
1994-09-14, by wenzelm
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
less
more
|
(0)
-480
+480
+1000
+3000
+10000
+30000
tip