Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+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.
added insort_insert
2010-03-06, by haftmann
added dom_option_map, map_of_map_keys
2010-03-06, by haftmann
added bulkload; tuned document
2010-03-06, by haftmann
merged
2010-03-06, by haftmann
merged
2010-03-05, by haftmann
moved lemma map_sorted_distinct_set_unique
2010-03-05, by haftmann
various refinements
2010-03-05, by haftmann
print message when finiteness of domain definition is detected
2010-03-05, by huffman
merged
2010-03-05, by huffman
skip coinduction proofs for indirect-recursive domain definitions
2010-03-05, by huffman
merged
2010-03-06, by wenzelm
introduce notion of 'decisive' deflations; use them to simplify proof script for rule 'finites'
2010-03-05, by huffman
add comment
2010-03-05, by huffman
move take_proofs-related stuff to a new section
2010-03-05, by huffman
remove dead code
2010-03-05, by huffman
tuned dead code;
2010-03-05, by wenzelm
use regular Proof.goal (which is what methods usually see) and prevent sledgehammer from crashing;
2010-03-05, by wenzelm
merged
2010-03-05, by wenzelm
fix proof script so 'domain foo = Foo foo' works
2010-03-05, by huffman
fix proof script so qdomain_isomorphism foo = foo' works
2010-03-05, by huffman
finish browser_info: invoke isabelle browser -b to ensure that the jar really exists;
2010-03-05, by wenzelm
isabelle browser -b: Admin/build only;
2010-03-05, by wenzelm
merged
2010-03-05, by huffman
skip proof of induction rule for indirect-recursive domain definitions
2010-03-05, by huffman
generalized inj_uminus; added strict_mono_imp_inj_on
2010-03-05, by hoelzl
merged
2010-03-05, by hoelzl
Add Lebesgue integral and probability space.
2010-03-04, by hoelzl
Supremum and Infimum on real intervals
2010-03-04, by hoelzl
Rewrite rules for images of minus of intervals
2010-03-04, by hoelzl
Add dense_le, dense_le_bounded, field_le_mult_one_interval.
2010-03-04, by hoelzl
Added natfloor and floor rules for multiplication and power.
2010-03-04, by hoelzl
Generalized setsum_cases
2010-03-04, by hoelzl
Added vimage_inter_cong
2010-03-04, by hoelzl
merged
2010-03-04, by huffman
move coinduction-related stuff into function prove_coindunction
2010-03-04, by huffman
add function add_qualified_simp_thm
2010-03-04, by huffman
generate lemma take_below, declare chain_take [simp]
2010-03-03, by huffman
switch to polyml-svn;
2010-03-04, by wenzelm
basic simplification of external_prover signature;
2010-03-04, by wenzelm
tuned;
2010-03-04, by wenzelm
renamed type_has_empty_sort to type_has_topsort -- {} is the full universal sort;
2010-03-04, by wenzelm
point to http://hginit.com/
2010-03-04, by wenzelm
Simplified a couple of proofs and corrected a comment
2010-03-04, by paulson
lemmas set_map_of_compr, map_of_inject_set
2010-03-04, by haftmann
merged
2010-03-03, by huffman
merged
2010-03-03, by huffman
remove dead code
2010-03-03, by huffman
add infix declarations
2010-03-03, by huffman
remove unnecessary theorem references
2010-03-03, by huffman
remove copy_of_dtyp from domain_axioms.ML
2010-03-03, by huffman
add_axioms returns an iso_info; add_theorems takes an iso_info as an argument
2010-03-03, by huffman
uniformly use variable names m and n in take-related lemmas; use export_without_context where appropriate
2010-03-03, by huffman
add function axiomatize_lub_take
2010-03-03, by huffman
move function mk_lub into holcf_library.ML
2010-03-03, by huffman
added extern_syntax;
2010-03-03, by wenzelm
merged
2010-03-03, by haftmann
more uniform naming conventions
2010-03-03, by haftmann
tuned whitespace
2010-03-03, by haftmann
restructured RBT theory
2010-03-03, by haftmann
stats for at-poly-test;
2010-03-03, by wenzelm
proper names for types cfun, sprod, ssum (cf. fa231b86cb1e);
2010-03-03, by wenzelm
merged, resolving some basic conflicts;
2010-03-03, by wenzelm
merged
2010-03-03, by krauss
updated patch for hgweb style: now applies to Mercurial 1.4.3 templates
2010-03-03, by krauss
fix fragile proof using old induction rule (cf. bdf8ad377877)
2010-03-03, by krauss
merged
2010-03-03, by hoelzl
replaced \<bullet> with inner
2010-03-02, by himmelma
tuned
2010-03-02, by himmelma
the ordering on real^1 is linear
2010-03-02, by himmelma
merged
2010-03-03, by bulwahn
made smlnj happy
2010-03-02, by bulwahn
adding depth to predicate compile quickcheck for mutabelle tests; removing obsolete references in predicate compile quickcheck
2010-03-02, by bulwahn
adding HOL-Mutabelle to tests
2010-03-02, by bulwahn
merged
2010-03-03, by haftmann
more explicit naming scheme
2010-03-03, by haftmann
merged
2010-03-02, by huffman
adapt to changed variable name in casedist theorem
2010-03-02, by huffman
remove dependency on domain_syntax.ML
2010-03-02, by huffman
update HOLCF makefile
2010-03-02, by huffman
simplify add_axioms function; remove obsolete domain_syntax.ML
2010-03-02, by huffman
proof scripts use variable name y for casedist
2010-03-02, by huffman
fixrec and repdef modules import holcf_library
2010-03-02, by huffman
use y as variable name in casedist, like datatype package
2010-03-02, by huffman
proper names for types cfun, sprod, ssum
2010-03-02, by huffman
variable name changed
2010-03-02, by huffman
fix proof script for take_apps so it works with indirect recursion
2010-03-02, by huffman
remove dead code
2010-03-02, by huffman
remove unused mixfix component from type cons
2010-03-02, by huffman
cleaned up, added type annotations
2010-03-02, by huffman
remove unused selector field from type arg
2010-03-02, by huffman
add_syntax no longer needs a definitional mode
2010-03-02, by huffman
add_axioms no longer needs a definitional mode
2010-03-02, by huffman
get rid of primes on thy variables
2010-03-02, by huffman
move definition of finiteness predicate into domain_take_proofs.ML
2010-03-02, by huffman
move take-related definitions and proofs to new module; simplify map_of_typ functions
2010-03-02, by huffman
remove map_tab argument to calc_axioms
2010-03-02, by huffman
remove dead code
2010-03-02, by huffman
merged
2010-03-02, by paulson
Slightly generalised a theorem
2010-03-02, by paulson
merged
2010-03-02, by paulson
merged
2010-02-19, by paulson
merged
2010-02-19, by paulson
merged
2010-02-05, by paulson
merged
2010-02-04, by paulson
merged
2010-02-02, by paulson
Correction of a tiny error
2010-02-02, by paulson
removed obsolete helper theory
2010-03-02, by krauss
merged
2010-03-02, by haftmann
dropped superfluous naming
2010-03-02, by haftmann
UNIV is not a logical constant
2010-03-02, by huffman
merged
2010-03-02, by huffman
re-enable bisim code, now in domain_theorems.ML
2010-03-02, by huffman
add missing rule to case_strict proof script
2010-03-02, by huffman
remove dead code
2010-03-02, by huffman
domain package no longer generates copy functions; all proofs use take functions instead
2010-03-02, by huffman
need to explicitly include REP_convex
2010-03-01, by huffman
add lemma lub_eq
2010-03-01, by huffman
add lemmas about ssum_map and sprod_map
2010-03-01, by huffman
generate take_take rules
2010-03-01, by huffman
add function define_take_functions
2010-03-01, by huffman
add missing strictify rule to proof script
2010-03-01, by huffman
qualify constructor names with type name
2010-03-01, by huffman
move definition of case combinator to domain_constructors.ML
2010-03-01, by huffman
remove dependence on Domain_Library
2010-03-01, by huffman
more uses of function get_vars
2010-03-01, by huffman
add functions get_vars, get_vars_avoiding
2010-03-01, by huffman
move proofs of pat_rews to domain_constructors.ML
2010-03-01, by huffman
add_domain_constructors takes iso_info record as argument
2010-02-28, by huffman
domain_isomorphism package proves deflation rules for map functions
2010-02-28, by huffman
store deflation thms for map functions in theory data
2010-02-28, by huffman
use function list_ccomb
2010-02-28, by huffman
add function define_const
2010-02-28, by huffman
fix infix declarations
2010-02-28, by huffman
move common functions into new file holcf_library.ML
2010-02-28, by huffman
get rid of incomplete pattern match warnings
2010-02-28, by huffman
move some powerdomain stuff into a new file
2010-02-28, by huffman
move case combinator syntax to domain_constructors.ML
2010-02-28, by huffman
remove redundant code
2010-02-28, by huffman
use correct syntax name for pattern combinator
2010-02-28, by huffman
fix output translation for Case syntax
2010-02-28, by huffman
move definition and syntax of pattern combinators into domain_constructors.ML
2010-02-28, by huffman
domain_isomorphism function returns iso_info record
2010-02-27, by huffman
move proofs of match_rews to domain_constructors.ML
2010-02-27, by huffman
remove dead code
2010-02-27, by huffman
removed dead code
2010-02-27, by huffman
register match functions from domain_constructors.ML
2010-02-27, by huffman
move definition of match combinators to domain_constructors.ML
2010-02-27, by huffman
move proofs of dis_rews to domain_constructors.ML; change dis_defins to iff-style
2010-02-27, by huffman
move definition of discriminators to domain_constructors.ML
2010-02-27, by huffman
move proofs of when_rews intro domain_constructors.ML
2010-02-27, by huffman
moved proofs of dist_les and dist_eqs to domain_constructors.ML
2010-02-27, by huffman
move proofs of casedist into domain_constructors.ML
2010-02-27, by huffman
move proofs of injects and inverts to domain_constructors.ML
2010-02-26, by huffman
reuse vars_of function
2010-02-26, by huffman
remove unnecessary stuff from argument to add_constructors function
2010-02-26, by huffman
reorder sections
2010-02-26, by huffman
move proof of con_rews into domain_constructor.ML
2010-02-26, by huffman
don't bother returning con_defs
2010-02-26, by huffman
move constructor-specific stuff to a separate function
2010-02-26, by huffman
replace prove_thm function
2010-02-26, by huffman
move proof of compactness rules into domain_constructors.ML
2010-02-26, by huffman
add some convenience functions
2010-02-26, by huffman
rewrite domain package code for selector functions
2010-02-25, by huffman
add function beta_of_def
2010-02-24, by huffman
reorganizing domain package code (in progress)
2010-02-24, by huffman
change domain package's treatment of variable names in theorems to be like datatype package
2010-02-24, by huffman
remove redundant lemma real_minus_half_eq
2010-02-24, by huffman
polished and converted some proofs to Isar style
2010-02-24, by huffman
killed more recdefs
2010-03-02, by krauss
tuned comment
2010-03-01, by krauss
repaired subscripts broken in d8d7d1b785af
2010-03-02, by haftmann
repaired definition (cf. d8d7d1b785af)
2010-03-02, by haftmann
authentic syntax for *all* logical entities;
2010-03-03, by wenzelm
mark_atoms: more precise treatment of SynExt.standard_token_markers vs. syntax consts;
2010-03-03, by wenzelm
notation for xsymbols (cf. ad039d29e01c);
2010-03-03, by wenzelm
"_type_prop" is syntax const -- recovered printing of OFCLASS;
2010-03-03, by wenzelm
removed unused external_names;
2010-03-03, by wenzelm
cleanup type translations;
2010-03-03, by wenzelm
adapted to authentic syntax -- actual types are verbatim;
2010-03-03, by wenzelm
authentic syntax for classes and type constructors;
2010-03-03, by wenzelm
more systematic mark/unmark operations;
2010-03-03, by wenzelm
proper (type_)notation;
2010-03-02, by wenzelm
proper antiquotations;
2010-03-02, by wenzelm
standard convention for syntax consts;
2010-03-02, by wenzelm
more precise scope of exception handler;
2010-03-02, by wenzelm
eliminated hard tabs;
2010-03-01, by wenzelm
tuned final whitespace;
2010-03-01, by wenzelm
repaired 'definition' (cf. d8d7d1b785af);
2010-03-01, by wenzelm
merged
2010-03-01, by wenzelm
more recdef (and old primrec) hunting
2010-03-01, by krauss
killed recdefs in HOL-Auth
2010-03-01, by krauss
merged
2010-03-01, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+1000
+3000
+10000
+30000
tip