merged
authornipkow
Thu, 07 Sep 2017 18:01:41 +0200
changeset 66612 84926115c2dd
parent 66609 a61181ffb1ce (diff)
parent 66611 c375b64a6c24 (current diff)
child 66613 db3969568560
merged
--- a/Admin/Release/CHECKLIST	Thu Sep 07 16:41:40 2017 +0200
+++ b/Admin/Release/CHECKLIST	Thu Sep 07 18:01:41 2017 +0200
@@ -93,12 +93,6 @@
   default = http://bitbucket.org/isabelle_project/isabelle-release
   default = ssh://hg@bitbucket.org/isabelle_project/isabelle-release
 
-- Admin/cronjob/self_update:
-  http://bitbucket.org/isabelle_project/isabelle-release
-
-- src/Pure/Admin/isabelle_cronjon.scala:
-  isabelle_repos_source = isabelle_release_source
-
 
 Post-release
 ============
--- a/src/HOL/Library/Monad_Syntax.thy	Thu Sep 07 16:41:40 2017 +0200
+++ b/src/HOL/Library/Monad_Syntax.thy	Thu Sep 07 18:01:41 2017 +0200
@@ -5,7 +5,7 @@
 section \<open>Monad notation for arbitrary types\<close>
 
 theory Monad_Syntax
-imports FSet "~~/src/Tools/Adhoc_Overloading"
+imports Main "~~/src/Tools/Adhoc_Overloading"
 begin
 
 text \<open>
@@ -61,6 +61,6 @@
   "(m \<then> n)" \<rightharpoonup> "(m \<bind> (\<lambda>_. n))"
 
 adhoc_overloading
-  bind Set.bind Predicate.bind Option.bind List.bind FSet.fbind
+  bind Set.bind Predicate.bind Option.bind List.bind
 
-end
\ No newline at end of file
+end
--- a/src/Pure/Admin/isabelle_cronjob.scala	Thu Sep 07 16:41:40 2017 +0200
+++ b/src/Pure/Admin/isabelle_cronjob.scala	Thu Sep 07 18:01:41 2017 +0200
@@ -23,9 +23,6 @@
   val isabelle_repos = main_dir + Path.explode("isabelle")
   val isabelle_repos_test = main_dir + Path.explode("isabelle-test")
   val afp_repos = main_dir + Path.explode("AFP")
-
-  val isabelle_dev_source = "http://isabelle.in.tum.de/repos/isabelle"
-  val isabelle_release_source = "http://bitbucket.org/isabelle_project/isabelle-release"
   val afp_source = "https://bitbucket.org/isa-afp/afp-devel"
 
   val jenkins_jobs = "identify" :: Jenkins.build_log_jobs
@@ -239,7 +236,7 @@
                 Build_History.remote_build_history(ssh,
                   isabelle_repos,
                   isabelle_repos.ext(r.host),
-                  isabelle_repos_source = isabelle_dev_source,
+                  isabelle_repos_source = "http://isabelle.in.tum.de/repos/isabelle",
                   isabelle_identifier = "cronjob_build_history",
                   self_update = self_update,
                   push_isabelle_home = push_isabelle_home,